| Commit message (Expand) | Author | Age |
* | Removing Exc_located and using the new exception enrichement | ppedrot | 2013-02-18 |
* | Revised the Ltac trace mechanism so that trace breaking due to | herbelin | 2013-02-17 |
* | Fixed #2970 (made that remember's eqn name is interpretable as an ltac var). | herbelin | 2013-01-29 |
* | Fixed synchronicity of filter with evar context in new_goal_with. | herbelin | 2013-01-29 |
* | Actually adding backtrace handling. | ppedrot | 2013-01-28 |
* | Uniformization of the "anomaly" command. | ppedrot | 2013-01-28 |
* | Added backtrace information to anomalies | ppedrot | 2013-01-28 |
* | New implementation of the conversion test, using normalization by evaluation to | mdenes | 2013-01-22 |
* | Yet a new reduction tactic in Coq : cbn | pboutill | 2012-12-21 |
* | Modulification of identifier | ppedrot | 2012-12-14 |
* | Moved Stringset and Stringmap to String namespace. | ppedrot | 2012-12-14 |
* | Monomorphization (tactics) | ppedrot | 2012-11-25 |
* | Taking into account the type of a definition (if it exists), and the | herbelin | 2012-11-17 |
* | Split Tacinterp in 3 files : Tacsubst, Tacintern and Tacinterp | letouzey | 2012-10-16 |
* | remove useless hidden_flag in TacMutual(Co)Fix | letouzey | 2012-10-06 |
* | cosmetic concerning interp of TacShowHyps | letouzey | 2012-10-06 |
* | remove Refiner.abstract_tactic and similar | letouzey | 2012-10-06 |
* | Adapt pieces of code needing -rectypes | letouzey | 2012-10-06 |
* | Clean-up : removal of Proof_type.tactic_expr | letouzey | 2012-10-06 |
* | Clean-up of proof_type.ml : no more Nested nor abstract_tactic_box | letouzey | 2012-10-06 |
* | Remove some more "open" and dead code thanks to OCaml4 warnings | letouzey | 2012-10-02 |
* | Added a new tactical infoH tac, that displays the names of hypothesis created... | courtieu | 2012-10-01 |
* | Some documentation and cleaning of CList and Util interfaces. | ppedrot | 2012-09-15 |
* | Moving Utils.list_* to a proper CList module, which includes stdlib | ppedrot | 2012-09-14 |
* | This patch removes unused "open" (automatically generated from | regisgia | 2012-09-14 |
* | The new ocaml compiler (4.00) has a lot of very cool warnings, | regisgia | 2012-09-14 |
* | Updating headers. | herbelin | 2012-08-08 |
* | Dump references in reduction tactics | pboutill | 2012-08-05 |
* | 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 |
* | Added an indirection with respect to Loc in Compat. As many [open Compat] | ppedrot | 2012-06-22 |
* | Replacing some str with strbrk | ppedrot | 2012-06-04 |
* | Cleaning Pp.ppnl use | ppedrot | 2012-06-01 |
* | Getting rid of Pp.msgnl and Pp.message. | ppedrot | 2012-06-01 |
* | More uniformisation in Pp.warn functions. | ppedrot | 2012-05-30 |
* | 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 |
* | 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 |
* | 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 |
* | Continuing r15045-15046 and r15055 (fixing bug #2732 about atomic | herbelin | 2012-03-20 |