aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* Many fixes in unification:Gravatar msozeau2009-05-20
* - Fixing declarative mode in presence of high use of Change_evars nodesGravatar herbelin2009-05-20
* Fix in canonical structure resolution: [check_conv_record] may returnGravatar msozeau2009-05-19
* Remove camlp4-specific exception handlingGravatar msozeau2009-05-19
* Minor unification changes:Gravatar msozeau2009-05-18
* - Allowing multiple calls to tactic fix with automatic generation ofGravatar herbelin2009-05-17
* (Tentative to) add Canonical Structure resolution to the regularGravatar msozeau2009-05-16
* Minor fixes in typeclasses:Gravatar msozeau2009-05-16
* Support for definition hooks in subtac.Gravatar msozeau2009-05-16
* Fix to my last notation patch: now fixpoint are correctly handled Gravatar vsiles2009-05-13
* minor bugfixes. CoqIde development will resume soon now ...Gravatar vgross2009-05-13
* micromega: proof compression bugfixGravatar fbesson2009-05-11
* - Addition of "Hint Resolve ->" and "Hint Resolve <-" continued: itGravatar herbelin2009-05-10
* - Adding "Hint Resolve ->" and "Hint Resolve <-" for declaration of equivalenceGravatar herbelin2009-05-09
* fix a bug in canonical structures (bug found and fixed by Cyril)Gravatar barras2009-05-09
* adds a theorem to reason at the level of ZGravatar bertot2009-05-07
* Improvements in typeclasses eauto and generalized rewriting:Gravatar msozeau2009-05-05
* Fix a small notation/scope bug:Gravatar vsiles2009-04-30
* More efficient handling of evars in Program Fixpoint commands.Gravatar msozeau2009-04-28
* Fixes for bugs in r12110:Gravatar msozeau2009-04-28
* _tags: lexer.ml4 now uses pa_macroGravatar letouzey2009-04-28
* Backporting 12112 from v8.2 branch to trunk (fixing documentation bugsGravatar herbelin2009-04-28
* Cleanup old eauto code.Gravatar msozeau2009-04-27
* - Implementation of a new typeclasses eauto procedure based on successGravatar msozeau2009-04-27
* - Fixed a little bug in previous commit (bad failure in case of unknown entry).Gravatar herbelin2009-04-27
* - Cleaning (unification of ML names, removal of obsolete code,Gravatar herbelin2009-04-27
* - Fixing #2090 (occur check missing when trying to solve evar-evar equation).Gravatar herbelin2009-04-25
* Report de la révision #12104 (Maj lien site web de Coq)Gravatar notin2009-04-24
* Backporting 12080 (fixing bug #2091 on bad rollback in the "where"Gravatar herbelin2009-04-24
* Fixing bug #2308 ("instantiate" tactic did not comply withGravatar herbelin2009-04-24
* - New cleaning phase for the entry points of pretyping.mlGravatar herbelin2009-04-24
* fixed CBV strategy: it was too eager on terms likeGravatar barras2009-04-21
* Rename [Morphism] into [Proper] and [respect] into [proper] to complyGravatar msozeau2009-04-21
* Fix test output mentionning an existential number that changed.Gravatar msozeau2009-04-20
* Fix wrong pattern in Morphisms. Fix bug scripts to reflect the fact thatGravatar msozeau2009-04-20
* Just export RelationClasses for [Equivalence] through Setoid.Gravatar msozeau2009-04-18
* Only export the notations of Morphism as well as Equivalence throughGravatar msozeau2009-04-17
* - Fix handling of clauses in setoid_rewrite to rewrite under bindersGravatar msozeau2009-04-17
* comparison functions on lists and arraysGravatar barras2009-04-16
* Fix bug #2089: correctly dealing with parameters and real arguments inGravatar msozeau2009-04-16
* Better Requires in Classes. Fix bug #2093: the code does not requireGravatar msozeau2009-04-16
* nouvelle version de la tactique groebner proposee par Loic:Gravatar barras2009-04-16
* Rewrite autorewrite to use a dnet indexed by the left-hand sides (orGravatar msozeau2009-04-14
* Add a combinator for rewriting given a list of terms and fix theGravatar msozeau2009-04-14
* Correction du patch -rectypes pour ocaml 3.10Gravatar vsiles2009-04-14
* Some additions in Max and Zmax. Unifiying list of statements and namesGravatar herbelin2009-04-14
* Fix and actually beautify the bug script to adapt to the new measureGravatar msozeau2009-04-14
* Rewrite of setoid_rewrite to modularize it based on proof-producingGravatar msozeau2009-04-13
* Fix premature optimisation in dependent induction: even variable args needGravatar msozeau2009-04-10
* Fix tauto no longer failing after commit 12077; appropriate errorGravatar herbelin2009-04-10