aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
Commit message (Expand)AuthorAge
* 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
* Yet a new reduction tactic in Coq : cbnGravatar pboutill2012-12-21
* Fixed a little inefficiency of "set/destruct" over a pattern. NowGravatar herbelin2012-12-18
* Modulification of identifierGravatar ppedrot2012-12-14
* Moved Intset and Intmap to Int namespace.Gravatar ppedrot2012-12-14
* Using library string functions.Gravatar ppedrot2012-12-13
* Monomorphization (tactics)Gravatar ppedrot2012-11-25
* Added a CString module.Gravatar ppedrot2012-11-13
* Monomorphized a lot of equalities over OCaml integers, thanks toGravatar ppedrot2012-11-08
* Remove some more "open" and dead code thanks to OCaml4 warningsGravatar letouzey2012-10-02
* More cleaning in CArray...Gravatar ppedrot2012-09-18
* Cleaning interface of Util.Gravatar ppedrot2012-09-18
* More cleaning on Utils and CList. Some parts of the code beingGravatar ppedrot2012-09-17
* As r15801: putting everything from Util.array_* to CArray.*.Gravatar ppedrot2012-09-14
* Moving Utils.list_* to a proper CList module, which includes stdlibGravatar ppedrot2012-09-14
* This patch removes unused "open" (automatically generated fromGravatar regisgia2012-09-14
* The new ocaml compiler (4.00) has a lot of very cool warnings,Gravatar regisgia2012-09-14
* Updating headers.Gravatar herbelin2012-08-08
* Reductionops refactoringGravatar pboutill2012-07-20
* induction/destruct : nicer syntax for generating equations (solves #2741)Gravatar letouzey2012-07-09
* ZArith + other : favor the use of modern names instead of compat notationsGravatar letouzey2012-07-05
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Let's try to avoid generating induction principles for records (wish #2693)Gravatar letouzey2012-06-01