aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
...
* Removing a bunch of generic equalities.Gravatar ppedrot2013-09-27
* Opacifying the type of strategies.Gravatar ppedrot2013-09-26
* Splitting Rewrite into a code part and a CAMLP4-dependent one.Gravatar ppedrot2013-09-26
* Removing useless evar-related stuff.Gravatar ppedrot2013-09-25
* Adding evar printing to debugger.Gravatar ppedrot2013-09-24
* Fixing ocamldebug compilation by adding thread linking.Gravatar ppedrot2013-09-24
* Fix name clash in "failure/inductive.v".Gravatar xclerc2013-09-20
* Merge "circular_subtyping?.v" tests into a single "circular_subtyping.v" test.Gravatar xclerc2013-09-20
* Merge "inductive?.v" tests into a single "inductive.v" test.Gravatar xclerc2013-09-20
* Get rid of "shouldsucceed" subdirectory by moving tests to parent directory.Gravatar xclerc2013-09-20
* Get rid of "shouldfail" subdirectory by moving tests to parent directory.Gravatar xclerc2013-09-20
* Wrong bug identifier.Gravatar xclerc2013-09-20
* Execute tests from the "bugs/closed" directory.Gravatar xclerc2013-09-20
* Update test for bug 2846 in order to use "Fail".Gravatar xclerc2013-09-20
* Use "Fail" rather than rely on exit code.Gravatar xclerc2013-09-20
* Uminus.v : prepare this test file for the use of FailGravatar letouzey2013-09-19
* universes-buraliforti-redef.v : repair a match after Pierre B. syntax changesGravatar letouzey2013-09-19
* Prettyp: avoid useless "let module"Gravatar letouzey2013-09-19
* Made the filename of compiled files explicit, i.e. add a ./ prefixGravatar ppedrot2013-09-19
* Get rid of the uses of deprecated OCaml elements (still remaining compatible ...Gravatar xclerc2013-09-19
* At least made the evar type opaque! There are still 5 remaining unsafeGravatar ppedrot2013-09-18
* Removing the last global evar generation in Term_dnet. The veryGravatar ppedrot2013-09-18
* Removing unused code from Term_dnet.Gravatar ppedrot2013-09-18
* Removing almost all new_untyped_evar, and a bunch of Evd.add.Gravatar ppedrot2013-09-18
* Taming the simpl evar hack that used to use negative evars.Gravatar ppedrot2013-09-18
* Slightly more compact representation of 'a substituted type,Gravatar ppedrot2013-09-14
* When Coq is reset-initialed by CoqIDE, do reset jobs countersGravatar gareuselesinge2013-09-13
* fix error reporting window size calculationGravatar gareuselesinge2013-09-13
* CoqIDE: new async error reporting window and slaves statusGravatar gareuselesinge2013-09-13
* STM pretty printer should never failGravatar gareuselesinge2013-09-13
* fix STM feeback on running jobsGravatar gareuselesinge2013-09-13
* Do no compage wg_Notebook terms with (=)Gravatar gareuselesinge2013-09-13
* Unplugging Autoinstance. The code is still here if someone wishesGravatar ppedrot2013-09-12
* CoqIDE: show number of proofs being checked in backgroundGravatar gareuselesinge2013-09-12
* Minimal implementation of `Shallow marshalling of LibGravatar gareuselesinge2013-09-12
* Unknown commands starting a proof were not setting the proof mode.Gravatar gareuselesinge2013-09-12
* Remove outdated commentGravatar gareuselesinge2013-09-12
* VernacList handling was lost in STM mergeGravatar gareuselesinge2013-09-12
* Fix bug in CStack introduced by refactoringGravatar gareuselesinge2013-09-12
* Temporary fix of emacs mode for ProofGeneralGravatar letouzey2013-09-10
* Change syntax of Hint Resolve to actually accept user-given priorities.Gravatar msozeau2013-09-07
* Moving Searchstack to CStack, and normalizing names a bit.Gravatar ppedrot2013-09-06
* Optimizing some evar_maps manipulation. In particular, using a [map] insteadGravatar ppedrot2013-09-05
* Documentation of Evd.Gravatar ppedrot2013-09-05
* Cleaning up of Evd. Extruding the tower of modules used to define evar_maps.Gravatar ppedrot2013-09-05
* More robust argument setter in CoqIDE. It does not crash anymore on badGravatar ppedrot2013-09-04
* Fixing some tests from the test-suite.Gravatar ppedrot2013-09-03
* Partly replacing list-based access functions in Evd. This is stillGravatar ppedrot2013-09-03
* Some cleanup in AutoGravatar ppedrot2013-09-03
* Removing more association lists in Constrintern.Gravatar ppedrot2013-09-02