aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
Commit message (Expand)AuthorAge
* 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
* Added support for option Local (at module level) in Tactic Notation.Gravatar herbelin2012-08-11
* Updating headers.Gravatar herbelin2012-08-08
* Bigint: new functions of_int and to_int, 2nd arg of pow in intGravatar letouzey2012-08-02
* Getting rid of the undocumented [complete] tactic, which wasGravatar ppedrot2012-07-19
* Re-allow Reset in compiled filesGravatar letouzey2012-07-11
* destruct: full compatibility with former _eqn syntaxGravatar letouzey2012-07-09
* 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
* Two adaptations after the changes of level of ->Gravatar letouzey2012-07-06
* A prototype implementation of a Print Namespace command.Gravatar aspiwack2012-07-06
* Fixes a bug in the parsing of the grammar entry dirpath which would,Gravatar aspiwack2012-07-06
* Notation: a new annotation "compat 8.x" extending "only parsing"Gravatar letouzey2012-07-05
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Internalization of pattern is done in two phases.Gravatar pboutill2012-06-14
* Fixing previous commit (something strange happened...)Gravatar ppedrot2012-06-04
* Replacing some str with strbrkGravatar ppedrot2012-06-04
* Added a color output to Coqtop.Gravatar ppedrot2012-06-04
* Getting rid of Pp.msgnl and Pp.message.Gravatar ppedrot2012-06-01
* Restore compatibility with camlp4 (some missing open Tok)Gravatar letouzey2012-05-30
* remove many excessive open Util & Errors in mli'sGravatar letouzey2012-05-29
* place all pretty-printing files in new dir printing/Gravatar letouzey2012-05-29
* Extend become a mli-only file in intf/Gravatar letouzey2012-05-29
* Avoid Dumpglob dependency on LexerGravatar letouzey2012-05-29
* place all files specific to camlp4 syntax extensions in grammar/Gravatar letouzey2012-05-29
* Split Egrammar into Egramml and EgramcoqGravatar letouzey2012-05-29
* No more Univ in grammar.cmaGravatar letouzey2012-05-29
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar letouzey2012-05-29
* Strongly reduce the dependencies of grammar.cma, modulo two hacksGravatar letouzey2012-05-29
* Basic stuff about constr_expr migrated from topconstr to constrexpr_opsGravatar letouzey2012-05-29
* Stuff about notation_constr (ex-aconstr) now in notation_ops.mlGravatar letouzey2012-05-29
* slim down a bit genarg.ml (pr_intro_pattern forgotten there)Gravatar letouzey2012-05-29
* Migrate the grammar entry about "Ltac" into g_vernac.ml4.Gravatar letouzey2012-05-29
* simplification in deps of some g_*.ml4Gravatar 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
* Decl_kinds becomes a pure mli file, remaining ops in new file kindops.mlGravatar letouzey2012-05-29
* Vernacexpr is now a mli-only file, locality stuff now in locality.mlGravatar letouzey2012-05-29
* Tactic unfold always asks for comma between names.Gravatar pboutill2012-05-09
* Partial revert of r15148 in order to compile with Camlp4Gravatar pboutill2012-04-27
* migrate g_obligations.ml4 in parsingGravatar letouzey2012-04-26
* Program: avoid staying in program mode after a failed Program commandGravatar letouzey2012-04-26
* 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
* Removed syntax BeginSubproof/EndSubproof. It has been replaced byGravatar aspiwack2012-04-13