| Commit message (Expand) | Author | Age |
* | Better treatment of error messages in rewrite (avoid use of Errors.print). | msozeau | 2012-07-10 |
* | The tactic remember now accepts a final eqn:H option (grant wish #2489) | letouzey | 2012-07-09 |
* | induction/destruct : nicer syntax for generating equations (solves #2741) | letouzey | 2012-07-09 |
* | Fix order of introduction of hints to preserve most-recent-first semantics. | msozeau | 2012-07-06 |
* | rewrite_db : a first attempt at using rewrite_strat for a quicker autorewrite | letouzey | 2012-07-05 |
* | ZArith + other : favor the use of modern names instead of compat notations | letouzey | 2012-07-05 |
* | Fixes in rewriting by strategies (almost ready to be documented!): | msozeau | 2012-07-05 |
* | Fixing previous commit. | ppedrot | 2012-06-28 |
* | Fixing info_auto / info_trivial display. | ppedrot | 2012-06-28 |
* | Added an indirection with respect to Loc in Compat. As many [open Compat] | ppedrot | 2012-06-22 |
* | Fix bug #2790: wrong handling of Set -> Prop -> Prop products in setoid rewri... | msozeau | 2012-06-19 |
* | Replacing some str with strbrk | ppedrot | 2012-06-04 |
* | Forward-port fixes from 8.4 (15358, 15353, 15333). | msozeau | 2012-06-04 |
* | More cleaning | ppedrot | 2012-06-01 |
* | Cleaning Pp.ppnl use | ppedrot | 2012-06-01 |
* | Getting rid of Pp.msgnl and Pp.message. | ppedrot | 2012-06-01 |
* | Let's try to avoid generating induction principles for records (wish #2693) | letouzey | 2012-06-01 |
* | tactic is_fix, akin to is_evar, is_hyp, is_ ... family | pboutill | 2012-05-31 |
* | Getting rid of Pp.msg | ppedrot | 2012-05-30 |
* | More uniformisation in Pp.warn functions. | ppedrot | 2012-05-30 |
* | remove many excessive open Util & Errors in mli's | letouzey | 2012-05-29 |
* | No need to have Refine amongst Hightactics.cm*a | letouzey | 2012-05-29 |
* | place all files specific to camlp4 syntax extensions in grammar/ | letouzey | 2012-05-29 |
* | global_reference migrated from Libnames to new Globnames, less deps in gramma... | letouzey | 2012-05-29 |
* | Basic stuff about constr_expr migrated from topconstr to constrexpr_ops | letouzey | 2012-05-29 |
* | slim down a bit genarg.ml (pr_intro_pattern forgotten there) | letouzey | 2012-05-29 |
* | Pattern as a mli-only file, operations in Patternops | letouzey | 2012-05-29 |
* | New files intf/constrexpr.mli and intf/notation_term.mli out of Topconstr | letouzey | 2012-05-29 |
* | Glob_term now mli-only, operations now in Glob_ops | letouzey | 2012-05-29 |
* | Tacexpr as a mli-only, the few functions there are now in Tacops | letouzey | 2012-05-29 |
* | locus.mli for occurrences+clauses, misctypes.mli for various little things | letouzey | 2012-05-29 |
* | Evar_kinds.mli containing former Evd.hole_kind, avoid deps on Evd | letouzey | 2012-05-29 |
* | Vernacexpr is now a mli-only file, locality stuff now in locality.ml | letouzey | 2012-05-29 |
* | Intuition: temporary(?) restore the unconditional unfolding of not | letouzey | 2012-05-15 |
* | remove undocumented and scarcely-used tactic auto decomp | letouzey | 2012-04-23 |
* | Corrects a (very) longstanding bug of tactics. As is were, tactic expecting | aspiwack | 2012-04-18 |
* | Adds the openconstr entry for tactic notations. | aspiwack | 2012-04-18 |
* | Better error message in tactic notations. | aspiwack | 2012-04-18 |
* | Remove the Dp plugin. | gmelquio | 2012-04-17 |
* | Fixing tauto "special" behavior on singleton types w/ 2 parameters (bug #2680). | herbelin | 2012-04-15 |
* | In "intro until" and its applications, be consistent when reduction is | herbelin | 2012-04-15 |
* | Remove print call that do not use the pp mechanism | pboutill | 2012-04-12 |
* | "A -> B" is a notation for "forall _ : A, B". | pboutill | 2012-04-12 |
* | info_trivial, info_auto, info_eauto, and debug (trivial|auto) | letouzey | 2012-03-30 |
* | Remove code of obsolete tactics : superauto, autotdb, cdhyp, dhyp, dconcl | letouzey | 2012-03-30 |
* | Fix interface of resolve_typeclasses: onlyargs -> with_goals: | msozeau | 2012-03-20 |
* | Continuing r15045-15046 and r15055 (fixing bug #2732 about atomic | herbelin | 2012-03-20 |
* | Fix bugs related to Program integration. | msozeau | 2012-03-19 |
* | Removing redundant entry int_nelist and removing extra space when | herbelin | 2012-03-18 |
* | Fixing bug #2732 (anomaly when using the tolerance for writing | herbelin | 2012-03-18 |