aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* Proof using: do not clear letins (unless they use a cleared var)Gravatar Enrico Tassi2014-12-29
* Use [Proof using] to make sure that [List.in_flat_map] doesn't grab too many ...Gravatar Arnaud Spiwack2014-12-28
* Call nf_constraints also when compiling directly to voGravatar Enrico Tassi2014-12-28
* Proof using: call "clear" to remove from sight the vars not selectedGravatar Enrico Tassi2014-12-28
* remove debug prints (leftover)Gravatar Enrico Tassi2014-12-28
* STM: check with the kernel proof terms on the worker tooGravatar Enrico Tassi2014-12-27
* STM: fix processing of errorsGravatar Enrico Tassi2014-12-27
* STM: module Pp is openGravatar Enrico Tassi2014-12-27
* proof_global: make it possible to call close_proof in a workerGravatar Enrico Tassi2014-12-27
* include test-suite/coqchk in the summary logGravatar Enrico Tassi2014-12-27
* universes_of_constant: do a proper set union of body and type univsGravatar Enrico Tassi2014-12-27
* Revert "Term: include a function to print terms"Gravatar Enrico Tassi2014-12-27
* new test for coqchkGravatar Enrico Tassi2014-12-26
* coqchk: flush the pp buffer from time to timeGravatar Enrico Tassi2014-12-26
* STM: do not call process_error twice (Close: 3880)Gravatar Enrico Tassi2014-12-26
* Call Evd.nf_constraints only on Univ Poly constantsGravatar Enrico Tassi2014-12-26
* STM: remove dead codeGravatar Enrico Tassi2014-12-26
* Term: include a function to print termsGravatar Enrico Tassi2014-12-26
* Document 6d5b56d971 (forbid Require inside modules).Gravatar Maxime Dénès2014-12-25
* Forbid Require inside interactive modules and module types.Gravatar Maxime Dénès2014-12-25
* Inlining Spawn.kill_if in the one place were it was actually used, thusGravatar Pierre-Marie Pédrot2014-12-25
* STM: cleanup code for AdmittedGravatar Enrico Tassi2014-12-23
* Vi2vo: fix handling of univ constraints coming from the bodyGravatar Enrico Tassi2014-12-23
* Minor modification of CHANGE.Gravatar Pierre Courtieu2014-12-23
* A global [gfail] tactic which works like [fail] except that it fails even if ...Gravatar Arnaud Spiwack2014-12-23
* Remove compatibility layer from Ltac's [fail].Gravatar Arnaud Spiwack2014-12-23
* Fix compilation error in some configurations.Gravatar Arnaud Spiwack2014-12-23
* Dead code in Univ.Gravatar Pierre-Marie Pédrot2014-12-21
* Win32: fix installerGravatar Enrico Tassi2014-12-19
* Install .v and .glob files tooGravatar Enrico Tassi2014-12-19
* Add a backtracking version of Ltac's [match].Gravatar Arnaud Spiwack2014-12-19
* When pretyping [uconstr] closures, don't use the local Ltac variable environm...Gravatar Arnaud Spiwack2014-12-19
* Fixing performance issue of checker validation.Gravatar Pierre-Marie Pédrot2014-12-19
* Fixing checker representation of values.Gravatar Pierre-Marie Pédrot2014-12-19
* update md5 sums to make "make check" workGravatar Enrico Tassi2014-12-19
* Fix sigsegv in checkerGravatar Enrico Tassi2014-12-19
* Better doc and a few fixes for Proof using.Gravatar Enrico Tassi2014-12-19
* Back to the preferred ?n1:=?n2 order of evar-evar unification which got accid...Gravatar Hugo Herbelin2014-12-19
* Fixing wrong notation level in #3295.Gravatar Hugo Herbelin2014-12-19
* Adds two lemmas about hderror to the List standard library.Gravatar Sébastien Hinderer2014-12-18
* Implement the nodup function on lists and prove associated results.Gravatar Sébastien Hinderer2014-12-18
* Lists: enhanced version of Seb's last commit on Exists/ForallGravatar Pierre Letouzey2014-12-18
* Lists: a few results on Exists and Forall and a bit of code cleanup.Gravatar Sébastien Hinderer2014-12-18
* Fixing checker representation of universe lists.Gravatar Pierre-Marie Pédrot2014-12-18
* Backporting the change in lists of universes to the checker.Gravatar Pierre-Marie Pédrot2014-12-18
* Cleaning up universe list implementation in Univ.Gravatar Pierre-Marie Pédrot2014-12-18
* Proof using: New vernacular to name sets of section variablesGravatar Enrico Tassi2014-12-18
* Bug fix (coq_makefile): Adding unix.cma and threads.cma dependencies for gram...Gravatar mlasson2014-12-18
* Fixed bad newlines in output for std output and emacs.Gravatar Pierre Courtieu2014-12-18
* Fix compilation with ocaml 4.0.0Gravatar Enrico Tassi2014-12-17