aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
Commit message (Expand)AuthorAge
* - Fixing bug #2084 (unification not checking sort constraints), hopingGravatar herbelin2009-04-08
* - Backport of 12053 (fixing parsing segfault bug #2087) and 12058 (fixingGravatar herbelin2009-04-08
* Rewrite of Program Fixpoint to overcome the previous limitations: Gravatar msozeau2009-03-28
* Remove unused mli filesGravatar letouzey2009-03-27
* Backport from v8.2 branch of 11986 (interpretation of quantifiedGravatar herbelin2009-03-22
* Many changes in the Makefile infrastructure + a beginning of ocamlbuildGravatar letouzey2009-03-20
* Directory 'contrib' renamed into 'plugins', to end confusion with archive of ...Gravatar letouzey2009-03-20
* - configure: affiche si le natdynlink est positionneGravatar barras2009-03-17
* Cleaning/improving the use of the "in" clause (e.g. "unfold foo in H at 4"Gravatar herbelin2009-03-16
* Better mechanism for loading initial pluginsGravatar letouzey2009-03-14
* Optionally list opaque constants in addition to axions/variables inGravatar msozeau2009-03-09
* Timeout message was not always displayedGravatar barras2009-03-04
* commande Timeout + compaction des traces de debug_tacticGravatar barras2009-03-04
* Backtrack sur la mémoïsation de nf_evar.Gravatar aspiwack2009-03-04
* =?utf-8?q?Tentative=20d'optimisation=20(en=20temps)=20sur=20[nf=5Fevar]=20et=...Gravatar aspiwack2009-02-27
* On remplace evar_map par evar_defs (seul evar_defs est désormais exporté Gravatar aspiwack2009-02-19
* Fix de divers petits problèmes d'installationGravatar notin2009-02-11
* Report des revisions #11826, #11828 et #11829 de v8.2 vers trunkGravatar notin2009-02-11
* Allow to turn contrib/subtac into a (nat)dynlink'able pluginGravatar letouzey2009-02-03
* Revert changes in pcoq functions to restore compatibility with contribsGravatar puech2009-01-26
* Petit nettoyage faisant suite au commit #11847 .Gravatar aspiwack2009-01-23
* Les records déclarés avec Record ne peuvent plus être récursifs (le Gravatar aspiwack2009-01-19
* - Structuring Numbers and fixing Setoid in stdlib's doc.Gravatar herbelin2009-01-19
* Backporting from v8.2 to trunk:Gravatar herbelin2009-01-18
* Getting rid of the previous implementation of setoid_rewrite which wasGravatar msozeau2009-01-18
* Last changes in type class syntax: Gravatar msozeau2009-01-18
* DISCLAIMERGravatar puech2009-01-17
* Fixing #1960 (xml bug with external on goal variable) and #1961Gravatar herbelin2009-01-14
* Fixing/improving management of uniform prefix Local and GlobalGravatar herbelin2009-01-14
* - Standardized prefix use of "Local"/"Global" modifiers as decided inGravatar herbelin2009-01-13
* - Deactivation of dynamic loading on Mac OS 10.5 (see bug #2024).Gravatar herbelin2009-01-11
* Conversion du fichier 'revision' en un fichier .ml + correction d'un bug dans...Gravatar notin2009-01-06
* Completed 11745 (move of jprover to user contribs) and cleaned 11743Gravatar herbelin2009-01-05
* Bug dans commit 11743Gravatar herbelin2009-01-04
* Fixed bugs #2001 (search_guard was overwriting the guard index givenGravatar herbelin2009-01-04
* Made the debugger work again:Gravatar herbelin2009-01-02
* Moved parts of Sign to Term. Unified some names (e.g. decomp_n_prod ->Gravatar herbelin2008-12-31
* - Added support for subterm matching in SearchAbout.Gravatar herbelin2008-12-29
* - Suppression date dans configure du trunkGravatar herbelin2008-12-26
* - coq_makefile: target install now respects the original tree structureGravatar herbelin2008-12-24
* Nettoyage des variables Coq et amélioration de coqmktop. LesGravatar notin2008-12-19
* Sequel of 11697: repair coqtop.byte when contribs are statically linked (+min...Gravatar letouzey2008-12-17
* Take advantage of natdynlink when available: almost all contribs become loada...Gravatar letouzey2008-12-16
* Generalized binding syntax overhaul: only two new binders: `() and `{},Gravatar msozeau2008-12-14
* About "apply in":Gravatar herbelin2008-12-09
* Correct handling of defined methods (let-ins) in instance declarations.Gravatar msozeau2008-12-04
* Inductive parameters: nicer doc examples and error messageGravatar letouzey2008-11-28
* - Synchronized subst_object with load_object (load_and_subst_objects)Gravatar herbelin2008-11-23
* Minor improvement to commit 11619Gravatar herbelin2008-11-23
* Fixed bug #2006 (type constraint on Record was not taken into account) +Gravatar herbelin2008-11-23