aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
Commit message (Expand)AuthorAge
* Writing [cut] tactic using the new monad.Gravatar Pierre-Marie Pédrot2013-12-02
* Fixing abstract tactic by using a dummy name out of a declared proof.Gravatar Pierre-Marie Pédrot2013-11-27
* Remove the Hiddentac module.Gravatar Arnaud Spiwack2013-11-25
* Remove some occurrences of obsolete operatorsGravatar Stephane Glondu2013-11-22
* Porting Tactics.assumption to the new engine.Gravatar ppedrot2013-11-08
* Refine now does iota reduction in addition to beta.Gravatar aspiwack2013-11-02
* Refine: Tactics.New.refine does beta-reduction.Gravatar aspiwack2013-11-02
* Made Proofview.Goal.hyps a named_context.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
* Fix behaviour of the refine tactic with respect to evars in types.Gravatar aspiwack2013-11-02
* Replaced monads.ml by an essentially equivalent proofview_gen.ml generated by...Gravatar aspiwack2013-11-02
* Removed spurious try/with in Proofview.Notation.(>>=) and (>>==).Gravatar aspiwack2013-11-02
* The tactic [admit] exits with the "unsafe" status.Gravatar aspiwack2013-11-02
* Cleanup of comments.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
* Conv_orable made functional and part of pre_envGravatar gareuselesinge2013-10-31
* More monomorphic List.mem + List.assoc + ...Gravatar letouzey2013-10-24
* cList: set-as-list functions are now with an explicit comparisonGravatar letouzey2013-10-23
* Moving side effects into evar_map. There was no reason to keep anotherGravatar ppedrot2013-10-05
* Removing a bunch of generic equalities.Gravatar ppedrot2013-09-27
* Get rid of the uses of deprecated OCaml elements (still remaining compatible ...Gravatar xclerc2013-09-19
* At least made the evar type opaque! There are still 5 remaining unsafeGravatar ppedrot2013-09-18
* Actually using the domain function for maps.Gravatar ppedrot2013-08-25
* Less "Coq" strings everywhereGravatar letouzey2013-08-22
* State Transaction MachineGravatar gareuselesinge2013-08-08
* Side effect free implementation of admit (Isabelle's oracle)Gravatar gareuselesinge2013-08-08
* Fixing #3062. Computation of the value of a fresh identifier wasGravatar ppedrot2013-08-04
* Removing useless casts between arrays and lists.Gravatar ppedrot2013-08-04
* Revising r16550 about providing intro patterns for applying injection:Gravatar herbelin2013-07-09
* Replacing lists by maps in matching interpretation.Gravatar ppedrot2013-06-05
* Now interpreting introduction patterns [x1 .. xn] and (x1,..,xn) as anGravatar herbelin2013-06-02
* Fixing buggy backtracking in "intros * pat" with failing "pat".Gravatar herbelin2013-06-02
* Setting "appcontext" as the default behaviour in Ltac matching.Gravatar ppedrot2013-05-28
* Use the Hook module here and there.Gravatar ppedrot2013-05-12
* A uniformization step around understand_* and interp_* functions.Gravatar herbelin2013-05-09
* Merging Context and Sign.Gravatar ppedrot2013-04-29
* Splitting Term into five unrelated interfaces:Gravatar ppedrot2013-04-29
* raise UnsafeSuccess -> feedback AddedAxiomGravatar gareuselesinge2013-04-25
* Minor code cleaning in CArray / CList.Gravatar ppedrot2013-03-23
* Using hnf instead of "intro H" for forcing reduction to a product.Gravatar herbelin2013-03-21
* Fixing an old pecularity of "red": head betaiota redexes are nowGravatar herbelin2013-03-21
* Restrict (try...with...) to avoid catching critical exn (part 10)Gravatar letouzey2013-03-13
* Added a Local Definition vernacular command. This type of definitionGravatar ppedrot2013-03-11
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* New implementation of the conversion test, using normalization by evaluation toGravatar mdenes2013-01-22