aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
...
* 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
* list_eq_dec now transparent (wish #2786)Gravatar letouzey2012-06-01
* Cancel the start of a proof if its init_tac fails (fix #2799)Gravatar letouzey2012-06-01
* tactic is_fix, akin to is_evar, is_hyp, is_ ... familyGravatar pboutill2012-05-31
* Coq_makefile bug for pluginsGravatar pboutill2012-05-31
* Functions *_beq aren't generated anymore, remove comments about themGravatar letouzey2012-05-30
* Adds Reference-Manual.out to .gitignoreGravatar letouzey2012-05-30
* Getting rid of Pp.msgGravatar ppedrot2012-05-30
* More uniformisation in Pp.warn functions.Gravatar ppedrot2012-05-30
* Restore compatibility with camlp4 (some missing open Tok)Gravatar letouzey2012-05-30
* Fixed an error display bug in CoqIDE.Gravatar ppedrot2012-05-29
* Re-allow Time Back* (cf discussion on coq-club)Gravatar letouzey2012-05-29
* Some documentation of recent changes concerning interfacesGravatar letouzey2012-05-29
* 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
* 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
* 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
* Glob_term: minor formattingGravatar 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
* Makefile.build: a rule for building grammar.dotGravatar letouzey2012-05-29
* Pfedit: two superfluous openGravatar 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
* Makefile: avoid too much exported vars (for win32)Gravatar letouzey2012-05-29
* Bugs revealed by playing with contribsGravatar pboutill2012-05-25
* Fix r15259 to get rid of bug 2783Gravatar pboutill2012-05-25
* Fixed #2769.Gravatar ppedrot2012-05-25
* Fixed #2789.Gravatar ppedrot2012-05-25
* Rewritten the handling of coq sentence processing, hopefully beingGravatar ppedrot2012-05-23
* CHANGES: fix a typo + an entry in the wrong sectionGravatar letouzey2012-05-23
* Fixed #2538 by adding an option to reset coqtop on tab switch, as suggested.Gravatar ppedrot2012-05-23
* Cleaned prerr_endline use.Gravatar ppedrot2012-05-23
* Revert copy/pasted function in to minilib thanks to clib.cmaGravatar pboutill2012-05-23