diff options
| author | aspiwack | 2013-11-02 15:34:01 +0000 |
|---|---|---|
| committer | aspiwack | 2013-11-02 15:34:01 +0000 |
| commit | 260965dcf60d793ba01110ace8945cf51ef6531f (patch) | |
| tree | d07323383e16bb5a63492e2721cf0502ba931716 /tactics/inv.mli | |
| parent | 328279514e65f47a689e2d23f132c43c86870c05 (diff) | |
Makes the new Proofview.tactic the basic type of Ltac.
On the compilation of Coq, we can see an increase of ~20% compile time on
my completely non-scientific tests. Hopefully this can be fixed.
There are a lot of low hanging fruits, but this is an iso-functionality commit.
With a few exceptions which were not necessary for the compilation of the theories:
- The declarative mode is not yet ported
- The timeout tactical is currently deactivated because it needs some subtle
I/O. The framework is ready to handle it, but I haven't done it yet.
- For much the same reason, the ltac debugger is unplugged. It will be more
difficult, but will eventually be back.
A few comments:
I occasionnally used a coercion from [unit Proofview.tactic] to the old
[Prooftype.tactic]. It should work smoothely, but loses any backtracking
information: the coerced tactics has at most one success.
- It is used in autorewrite (it shouldn't be a problem there). Autorewrite's
code is fairly old and tricky
- It is used in eauto, mostly for "Hint Extern". It may be an issue as time goes
as we might want to have various success in a "Hint Extern". But it would
require a heavy port of eauto.ml4
- It is used in typeclass eauto, but with a little help from Matthieu, it should
be easy to port the whole thing to the new tactic engine, actually simplifying
the code.
- It is used in fourier. I believe it to be inocuous.
- It is used in firstorder and congruence. I think it's ok. Their code is
somewhat intricate and I'm not sure they would be easy to actually port.
- It is used heavily in Function. And honestly, I have no idea whether it can do
harm or not.
Updates:
(11 June 2013) Pierre-Marie Pédrot contributed the rebase over his new stream based
architecture for Ltac matching (r16533), which avoid painfully and expensively
working around the exception-throwing control flow of the previous API.
(11 October 2013) Rebasing over recent commits (somewhere in r16721-r16730)
rendered a major bug in my implementation of Tacticals.New.tclREPEAT_MAIN
apparent. It caused Field_theory.v to loop. The bug made rewrite !lemma,
rewrite ?lemma and autorewrite incorrect (tclREPEAT_MAIN was essentially
tclREPEAT, causing rewrites to be tried in the side-conditions of conditional
rewrites as well). The new implementation makes Coq faster, but it is
pretty much impossible to tell if it is significant at all.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16967 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/inv.mli')
| -rw-r--r-- | tactics/inv.mli | 22 |
1 files changed, 11 insertions, 11 deletions
diff --git a/tactics/inv.mli b/tactics/inv.mli index 52db199ee0..9491b7d7b9 100644 --- a/tactics/inv.mli +++ b/tactics/inv.mli @@ -19,24 +19,24 @@ type inversion_status = Dep of constr option | NoDep val inv_gen : bool -> inversion_kind -> inversion_status -> - intro_pattern_expr located option -> quantified_hypothesis -> tactic + intro_pattern_expr located option -> quantified_hypothesis -> unit Proofview.tactic val invIn_gen : inversion_kind -> intro_pattern_expr located option -> Id.t list -> - quantified_hypothesis -> tactic + quantified_hypothesis -> unit Proofview.tactic val inv_clause : inversion_kind -> intro_pattern_expr located option -> Id.t list -> - quantified_hypothesis -> tactic + quantified_hypothesis -> unit Proofview.tactic val inv : inversion_kind -> intro_pattern_expr located option -> - quantified_hypothesis -> tactic + quantified_hypothesis -> unit Proofview.tactic val dinv : inversion_kind -> constr option -> - intro_pattern_expr located option -> quantified_hypothesis -> tactic + intro_pattern_expr located option -> quantified_hypothesis -> unit Proofview.tactic -val half_inv_tac : Id.t -> tactic -val inv_tac : Id.t -> tactic -val inv_clear_tac : Id.t -> tactic -val half_dinv_tac : Id.t -> tactic -val dinv_tac : Id.t -> tactic -val dinv_clear_tac : Id.t -> tactic +val half_inv_tac : Id.t -> unit Proofview.tactic +val inv_tac : Id.t -> unit Proofview.tactic +val inv_clear_tac : Id.t -> unit Proofview.tactic +val half_dinv_tac : Id.t -> unit Proofview.tactic +val dinv_tac : Id.t -> unit Proofview.tactic +val dinv_clear_tac : Id.t -> unit Proofview.tactic |
