aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/extratactics.ml4
Commit message (Expand)AuthorAge
* Adding generic solvers to term holes. For now, no resolution mechanism norGravatar Pierre-Marie Pédrot2013-11-27
* Remove the Hiddentac module.Gravatar Arnaud Spiwack2013-11-25
* Doc: solve the bad interaction between Declare Implicit Tactic and refine.Gravatar aspiwack2013-11-02
* Refine: Tactics.New.refine does beta-reduction.Gravatar aspiwack2013-11-02
* Adds a tactic give_up.Gravatar aspiwack2013-11-02
* A tactic shelve_unifiable.Gravatar aspiwack2013-11-02
* Adds a shelve tactic.Gravatar aspiwack2013-11-02
* Refine does beta-reductions.Gravatar aspiwack2013-11-02
* Less use of the list-based interface for goal-bound tactics.Gravatar aspiwack2013-11-02
* Tachmach.New is now in Proofview.Goal.enter style.Gravatar aspiwack2013-11-02
* More Proofview.Goal.enter.Gravatar aspiwack2013-11-02
* Clean up a warning.Gravatar aspiwack2013-11-02
* The tactic [admit] exits with the "unsafe" status.Gravatar aspiwack2013-11-02
* A whole new implemenation of the refine tactic.Gravatar aspiwack2013-11-02
* Clean-up: removed redundant notations (>>-) and (>>--) from Proofview.Notations.Gravatar aspiwack2013-11-02
* Getting rid of Goal.here, and all the related exceptions and combinators.Gravatar aspiwack2013-11-02
* Makes the new Proofview.tactic the basic type of Ltac.Gravatar aspiwack2013-11-02
* Moving side effects into evar_map. There was no reason to keep anotherGravatar ppedrot2013-10-05
* Vernac classification streamlined (handles VERNAC EXTEND)Gravatar gareuselesinge2013-08-08
* State Transaction MachineGravatar gareuselesinge2013-08-08
* Start documenting new [rewrite_strat] tactic that applies rewritingGravatar msozeau2013-06-04
* Making the behavior of "injection ... as ..." more natural:Gravatar herbelin2013-06-02
* Granting wish #3014:Gravatar ppedrot2013-05-12
* Splitting Term into five unrelated interfaces:Gravatar ppedrot2013-04-29
* code simplifications concerning SummaryGravatar letouzey2013-04-22
* Restrict (try...with...) to avoid catching critical exn (part 13)Gravatar letouzey2013-03-13
* Removing Exc_located and using the new exception enrichementGravatar ppedrot2013-02-18
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* Modulification of identifierGravatar ppedrot2012-12-14
* Finish patch for Hint Resolve, stopping to generate new constant names forGravatar msozeau2012-12-08
* Monomorphization (tactics)Gravatar ppedrot2012-11-25
* Change Hint Resolve, Immediate to take a global reference as argumentGravatar msozeau2012-10-26
* Continue killing hidden tactics : no more generated h_xxxGravatar letouzey2012-10-15
* Remove some more "open" and dead code thanks to OCaml4 warningsGravatar letouzey2012-10-02
* As r15801: putting everything from Util.array_* to CArray.*.Gravatar ppedrot2012-09-14
* Updating headers.Gravatar herbelin2012-08-08
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Getting rid of Pp.msgnl and Pp.message.Gravatar ppedrot2012-06-01
* tactic is_fix, akin to is_evar, is_hyp, is_ ... familyGravatar pboutill2012-05-31
* Getting rid of Pp.msgGravatar ppedrot2012-05-30
* place all files specific to camlp4 syntax extensions in grammar/Gravatar letouzey2012-05-29
* Basic stuff about constr_expr migrated from topconstr to constrexpr_opsGravatar letouzey2012-05-29
* Glob_term now mli-only, operations now in Glob_opsGravatar letouzey2012-05-29
* locus.mli for occurrences+clauses, misctypes.mli for various little thingsGravatar letouzey2012-05-29
* Evar_kinds.mli containing former Evd.hole_kind, avoid deps on EvdGravatar letouzey2012-05-29
* Remove the Dp plugin.Gravatar gmelquio2012-04-17
* Second step of integration of Program:Gravatar msozeau2012-03-14
* Noise for nothingGravatar pboutill2012-03-02
* A "Grab Existential Variables" to transform the unresolved evars at the end o...Gravatar aspiwack2012-02-07
* Merge subinstances branch by me and Tom Prince.Gravatar msozeau2011-11-17