| Commit message (Expand) | Author | Age |
* | Legacy Ring and Legacy Field migrated to contribs | letouzey | 2012-07-05 |
* | rewrite_db : a first attempt at using rewrite_strat for a quicker autorewrite | letouzey | 2012-07-05 |
* | More cleanup in Ring_polynom and EnvRing | letouzey | 2012-07-05 |
* | Kills the useless tactic annotations "in |- *" | letouzey | 2012-07-05 |
* | Open Local Scope ---> Local Open Scope, same with Notation and alii | letouzey | 2012-07-05 |
* | ZArith + other : favor the use of modern names instead of compat notations | letouzey | 2012-07-05 |
* | Cleaning opening of the standard List module. | ppedrot | 2012-06-28 |
* | Replace nat indices with positive one in Btauto. | ppedrot | 2012-06-28 |
* | Added an indirection with respect to Loc in Compat. As many [open Compat] | ppedrot | 2012-06-22 |
* | Internalization of pattern is done in two phases. | pboutill | 2012-06-14 |
* | Changed encoding from ISO-8859-1 to UTF-8 for some remaining gallina files. | ppedrot | 2012-06-12 |
* | 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 |
* | 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 |
* | 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 |
* | Stuff about notation_constr (ex-aconstr) now in notation_ops.ml | 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 |
* | Decl_kinds becomes a pure mli file, remaining ops in new file kindops.ml | letouzey | 2012-05-29 |
* | Vernacexpr is now a mli-only file, locality stuff now in locality.ml | letouzey | 2012-05-29 |
* | Fix ocamlbuild compilation: remove subtac from *.itarget | letouzey | 2012-04-23 |
* | correct abort in Function when a proof of inversion fails | letouzey | 2012-04-23 |
* | Corrects a (very) longstanding bug of tactics. As is were, tactic expecting | aspiwack | 2012-04-18 |
* | Remove the Dp plugin. | gmelquio | 2012-04-17 |
* | "A -> B" is a notation for "forall _ : A, B". | pboutill | 2012-04-12 |
* | lib directory is cut in 2 cma. | pboutill | 2012-04-12 |
* | remove plugins/subtac/subtac.ml reintroduced by mistaked in a previous commit | letouzey | 2012-04-12 |
* | info_trivial, info_auto, info_eauto, and debug (trivial|auto) | letouzey | 2012-03-30 |
* | Module names and constant/inductive names are now in two separate namespaces | letouzey | 2012-03-26 |
* | A unified backtrack mechanism, with a basic "Show Script" as side-effect | letouzey | 2012-03-23 |
* | Fixing alpha-conversion bug #2723 introduced in r12485-12486. | herbelin | 2012-03-20 |
* | Fixing bug #2732 (anomaly when using the tolerance for writing | herbelin | 2012-03-18 |
* | Fix merge. | msozeau | 2012-03-14 |
* | Revise API of understand_ltac to be parameterized by a flag for resolution of... | msozeau | 2012-03-14 |
* | Final part of moving Program code inside the main code. Adapted add_definitio... | msozeau | 2012-03-14 |
* | Integrated obligations/eterm and program well-founded fixpoint building to to... | msozeau | 2012-03-14 |
* | Everything compiles again. | msozeau | 2012-03-14 |
* | Second step of integration of Program: | msozeau | 2012-03-14 |
* | Remove support for "abstract typing constraints" that requires unicity of sol... | msozeau | 2012-03-14 |
* | Glob_term.predicate_pattern: No number of parameters with letins. | pboutill | 2012-03-02 |