aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
Commit message (Expand)AuthorAge
* Partial revert of Yann commit in order to use CLib.List when openingGravatar 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
* fast bitwise operations (lor,land,lxor) on int31 and BigNGravatar letouzey2012-08-11
* Updating headers.Gravatar herbelin2012-08-08
* Dump references in reduction tacticsGravatar pboutill2012-08-05
* Dump referencesGravatar pboutill2012-08-05
* Reductionops refactoringGravatar pboutill2012-07-20
* Fix typeclass error handling which was sometimes raising a Failure ("hd").Gravatar msozeau2012-07-11
* Better treatment of error messages in rewrite (avoid use of Errors.print).Gravatar msozeau2012-07-10
* The tactic remember now accepts a final eqn:H option (grant wish #2489)Gravatar letouzey2012-07-09
* induction/destruct : nicer syntax for generating equations (solves #2741)Gravatar letouzey2012-07-09
* Fix order of introduction of hints to preserve most-recent-first semantics.Gravatar msozeau2012-07-06
* rewrite_db : a first attempt at using rewrite_strat for a quicker autorewriteGravatar letouzey2012-07-05
* ZArith + other : favor the use of modern names instead of compat notationsGravatar letouzey2012-07-05
* Fixes in rewriting by strategies (almost ready to be documented!):Gravatar msozeau2012-07-05
* Fixing previous commit.Gravatar ppedrot2012-06-28
* Fixing info_auto / info_trivial display.Gravatar ppedrot2012-06-28
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Fix bug #2790: wrong handling of Set -> Prop -> Prop products in setoid rewri...Gravatar msozeau2012-06-19
* Replacing some str with strbrkGravatar ppedrot2012-06-04
* Forward-port fixes from 8.4 (15358, 15353, 15333).Gravatar msozeau2012-06-04
* More cleaningGravatar ppedrot2012-06-01
* Cleaning Pp.ppnl useGravatar ppedrot2012-06-01
* Getting rid of Pp.msgnl and Pp.message.Gravatar ppedrot2012-06-01
* Let's try to avoid generating induction principles for records (wish #2693)Gravatar letouzey2012-06-01
* tactic is_fix, akin to is_evar, is_hyp, is_ ... familyGravatar pboutill2012-05-31
* Getting rid of Pp.msgGravatar ppedrot2012-05-30
* More uniformisation in Pp.warn functions.Gravatar ppedrot2012-05-30
* remove many excessive open Util & Errors in mli'sGravatar letouzey2012-05-29
* No need to have Refine amongst Hightactics.cm*aGravatar letouzey2012-05-29
* place all files specific to camlp4 syntax extensions in grammar/Gravatar letouzey2012-05-29
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar letouzey2012-05-29
* Basic stuff about constr_expr migrated from topconstr to constrexpr_opsGravatar letouzey2012-05-29
* slim down a bit genarg.ml (pr_intro_pattern forgotten there)Gravatar letouzey2012-05-29
* Pattern as a mli-only file, operations in PatternopsGravatar letouzey2012-05-29
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar letouzey2012-05-29
* Glob_term now mli-only, operations now in Glob_opsGravatar letouzey2012-05-29
* Tacexpr as a mli-only, the few functions there are now in TacopsGravatar 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
* Vernacexpr is now a mli-only file, locality stuff now in locality.mlGravatar letouzey2012-05-29
* Intuition: temporary(?) restore the unconditional unfolding of notGravatar letouzey2012-05-15
* remove undocumented and scarcely-used tactic auto decompGravatar letouzey2012-04-23
* Corrects a (very) longstanding bug of tactics. As is were, tactic expectingGravatar aspiwack2012-04-18
* Adds the openconstr entry for tactic notations.Gravatar aspiwack2012-04-18
* Better error message in tactic notations.Gravatar aspiwack2012-04-18
* Remove the Dp plugin.Gravatar gmelquio2012-04-17
* Fixing tauto "special" behavior on singleton types w/ 2 parameters (bug #2680).Gravatar herbelin2012-04-15