aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib
Commit message (Expand)AuthorAge
* Extraction: better dependency computation (after optimisations)Gravatar letouzey2008-07-20
* Rétablissement de l'option -dump-glob de coq top et de l'option -glob-from d...Gravatar notin2008-07-18
* Modification rapide du message d'erreur lorsqu'un _ ne peut êtreGravatar herbelin2008-07-18
* ROmega : make it work even if no Require Import ZArith has been doneGravatar letouzey2008-07-16
* Micromega: doc + test-suite updateGravatar fbesson2008-07-07
* Fix bug #1899: no more strange notations for Qge and QgtGravatar letouzey2008-07-04
* Correct a bug in the coercion code where we did not go under constantsGravatar msozeau2008-07-02
* Improved robustness of micromega parser. Proof search of Micromega test-suite...Gravatar fbesson2008-07-02
* Various bug fixes in type classes and subtac:Gravatar msozeau2008-07-01
* Correction bug "parser" suite changement syntaxeGravatar herbelin2008-06-29
* Enhanced discrimination nets implementation, which can now work withGravatar msozeau2008-06-27
* Création du fichier dumpglob.ml, qui rassemble les fonctions de globalisatio...Gravatar notin2008-06-25
* Micromega : bugs fixes - renaming of tactics - documentationGravatar fbesson2008-06-25
* Rename obligations_tactic to obligation_tactic and fix bugs #1893.Gravatar msozeau2008-06-22
* Code cleanup in typeclasses, remove dead and duplicated code.Gravatar msozeau2008-06-21
* - Implantation de la suggestion 1873 sur discriminate. Au final,Gravatar herbelin2008-06-21
* Various improvements in handling of evars in general and typingGravatar msozeau2008-06-21
* Little fixes: print unbound variable in error message (patch by SamuelGravatar msozeau2008-06-19
* Improvements in subtac:Gravatar msozeau2008-06-18
* Compatibility fixes (Add Setoid bug and accidental introduction of aGravatar msozeau2008-06-18
* Cleanup in subtac_cases, preparing to use improvements on return predicateGravatar msozeau2008-06-17
* Add possibility to match on defined hypotheses, using brackets toGravatar msozeau2008-06-16
* Correction parser révélé par test-suiteGravatar herbelin2008-06-12
* - Officialisation de la notation "pattern c at -1" (cf wish 1798 sur coq-bugs)Gravatar herbelin2008-06-10
* Suppression de la dépendance de Micromega envers Coq.Reals.Reals. Corrige le...Gravatar notin2008-06-10
* - Extension de "generalize" en "generalize c as id at occs".Gravatar herbelin2008-06-08
* Fixes incorrect handling of existing existentials variables inGravatar msozeau2008-06-03
* Minor bug correction in recdefGravatar jforest2008-06-02
* Improvements on coqdoc by adding more information into .globGravatar msozeau2008-05-30
* - Fix bug #1858, Hint Unfold calling the wrong locate function.Gravatar msozeau2008-05-23
* Strategy commands are now exportedGravatar barras2008-05-22
* refined the conversion oracleGravatar barras2008-05-21
* Corrections d'erreurs rapportées par Frédéric Besson sur le précédentGravatar herbelin2008-05-20
* Intégration de micromega ("omicron" pour fourier et sa variante sur Z,Gravatar herbelin2008-05-19
* Various fixes:Gravatar msozeau2008-05-15
* - Fix bug related to indices of fixpoints.Gravatar msozeau2008-05-13
* debug et nouvelles commandes Dp_prelude et Dp_predefinedGravatar filliatr2008-05-13
* - Add -unicode flag to coqtop (sets Flags.unicode_syntax). Used toGravatar msozeau2008-05-12
* - Cleanup parsing of binders, reducing to a single production for allGravatar msozeau2008-05-11
* Backtrack sur la mise à disposition en standard de la notation [ x ; ... ; y ]Gravatar herbelin2008-05-09
* Autre oubli de la révision 10904Gravatar herbelin2008-05-08
* export Extract_env.mono_environment in the mli Gravatar letouzey2008-05-07
* Postpone the search for the recursive argument index from the user givenGravatar msozeau2008-05-06
* Mise en place d'un algorithme d'inversion des contraintes de type lorsGravatar herbelin2008-05-05
* Clarification de l'ordre d'interprétation des variables dans ltac. EnGravatar herbelin2008-05-01
* Ajout notation [ x ; ... ; y ] dans list_scope. Changement de laGravatar herbelin2008-04-29
* Suppression de la partie ML de la contrib correctness. Les fichiersGravatar herbelin2008-04-29
* menage dans funind + deplaceemnt de recdef dans funindGravatar jforest2008-04-28
* Backtrack on using metas eagerly in auto, only done in "new auto" forGravatar msozeau2008-04-28
* Correction du bug des types singletons pas sous-type de SetGravatar herbelin2008-04-27