aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
Commit message (Expand)AuthorAge
* Getting rid of Pp.msgGravatar ppedrot2012-05-30
* More uniformisation in Pp.warn functions.Gravatar ppedrot2012-05-30
* Re-allow Time Back* (cf discussion on coq-club)Gravatar 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
* 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
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar 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
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar 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
* Revert copy/pasted function in to minilib thanks to clib.cmaGravatar pboutill2012-05-23
* Added a SearchAbout-like primitive in coqtop interface.Gravatar ppedrot2012-05-13
* Added an interface primitive to ask coqtop for its internal versions.Gravatar ppedrot2012-05-13
* Slightly modified the coqtop interface by adding an identifier inGravatar ppedrot2012-05-11
* Added an interface call to exit Coqtop nicely.Gravatar ppedrot2012-05-02
* Implicit arguments of Definition are taken from the type when given by the user.Gravatar 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
* correct abort in Function when a proof of inversion failsGravatar letouzey2012-04-23
* Supporting optional byte-mark order in utf-8 files (bug #2757).Gravatar herbelin2012-04-19
* Corrects a (very) longstanding bug of tactics. As is were, tactic expectingGravatar aspiwack2012-04-18
* Bug 2733 : { } implicits and FixpointsGravatar pboutill2012-04-17
* Better error message when defining recursive records with Record orGravatar aspiwack2012-04-13
* Remove print call that do not use the pp mechanismGravatar pboutill2012-04-12
* lib directory is cut in 2 cma.Gravatar pboutill2012-04-12
* Relax uniform inheritance conditionGravatar gareuselesinge2012-04-05
* Added a command "Unfocused" which returns an error when the proof isGravatar aspiwack2012-03-30
* Remove code of obsolete tactics : superauto, autotdb, cdhyp, dhyp, dconclGravatar letouzey2012-03-30
* Slight change in the semantics of arguments scopes: scopes can noGravatar herbelin2012-03-26
* A unified backtrack mechanism, with a basic "Show Script" as side-effectGravatar letouzey2012-03-23
* Remove undocumented command "Delete foo"Gravatar letouzey2012-03-23
* Remove old proof-managment commands Suspend/ResumeGravatar letouzey2012-03-23
* Fix interface of resolve_typeclasses: onlyargs -> with_goals:Gravatar msozeau2012-03-20
* Fixing alpha-conversion bug #2723 introduced in r12485-12486.Gravatar herbelin2012-03-20
* Continuing r15045-15046 and r15055 (fixing bug #2732 about atomicGravatar herbelin2012-03-20
* Force Check (which, from 8.4beta, accepts unresolved evars) to howeverGravatar herbelin2012-03-20
* Fix bugs related to Program integration.Gravatar msozeau2012-03-19
* Fixing bug #2732 (anomaly when using the tolerance for writingGravatar herbelin2012-03-18
* Fix merge and add missing file.Gravatar msozeau2012-03-14
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14
* Integrated obligations/eterm and program well-founded fixpoint building to to...Gravatar msozeau2012-03-14
* Everything compiles again.Gravatar msozeau2012-03-14
* Second step of integration of Program:Gravatar msozeau2012-03-14
* Noise for nothingGravatar pboutill2012-03-02