aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernacexpr.ml
Commit message (Expand)AuthorAge
...
* Strategy commands are now exportedGravatar barras2008-05-22
* refined the conversion oracleGravatar barras2008-05-21
* - 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
* ** Efficacité, bugs, robustesse CoqIDE **Gravatar herbelin2008-05-08
* Ajout de "Theorem id1 : t1 ... with idn : tn" pour partager la preuveGravatar herbelin2008-04-25
* Prise en compte des coercions dans les clauses "with" même si le typeGravatar herbelin2008-04-23
* - Add "Global" modifier for instances inside sections with the usualGravatar msozeau2008-04-15
* Ajout d'abbréviations/notations paramétriquesGravatar herbelin2008-03-30
* Various fixes on typeclasses:Gravatar msozeau2008-03-27
* Syntax changes in typeclasses, remove "?" for usual implicit argumentsGravatar msozeau2008-03-06
* Merge with lmamane's private branch:Gravatar lmamane2008-02-22
* Beaoucoup de changements dans la representation interne des modules.Gravatar soubiran2008-02-01
* Support for substructures in classes using :> notationGravatar msozeau2008-01-30
* Change notation for setoid inequality, coerce objects before comparing them. ...Gravatar msozeau2008-01-18
* Generalize instance declarations to any context, better name handling. Add ho...Gravatar msozeau2008-01-15
* Cleaner quantifiers for type classes, breaks clrewrite for the moment but imp...Gravatar msozeau2008-01-07
* Merged revisions 10358-10362,10365,10371-10373,10377,10383-10384,10394-10395,...Gravatar msozeau2007-12-31
* Nettoyage de Print Assumptions :Gravatar aspiwack2007-11-09
* Modification of the Scheme command.Gravatar vsiles2007-09-28
* Modification of VernacScheme to handle a new scheme: Equality (equality inGravatar vsiles2007-05-25
* Processor integers + Print assumption (see coqdev mailing list for the Gravatar aspiwack2007-05-11
* Nouveaux changements autour des implicites (notamment suite àGravatar herbelin2007-05-06
* New keyword "Inline" for Parameters and Axioms for automatic Gravatar soubiran2007-04-25
* Achèvement commit 9677 (suppression résidu v7 dans PrintGrammar)Gravatar herbelin2007-02-24
* Nouvelle approche pour le discharge modulaireGravatar herbelin2007-01-10
* Addition of a "Combined Scheme" vernacular command for building the conjuncti...Gravatar msozeau2006-12-23
* Declarative Proof Language: main commitGravatar corbinea2006-09-20
* Ajout possibilité clause "where" dans co-points fixes Gravatar herbelin2006-09-01
* Branchement de 'Debug On/Off' sur le mécanisme standard d'option et donc, re...Gravatar herbelin2006-07-05
* Suppression code pour hints nommés à la V7 (voire à la V6...)Gravatar herbelin2006-01-28
* Renommage des Pp*new en Pp* (et déplacement dans parsing); renommage des G_*...Gravatar herbelin2005-12-26
* Suppression des parseurs et printeurs v7; suppression du traducteur (mécanis...Gravatar herbelin2005-12-26
* Simplifification de vernac_expr li l'abandon du traducteurGravatar herbelin2005-12-23
* - debugging og "Show Intros": no line breaking + fresh idsGravatar coq2005-11-08
* New command: "Print Ltac qualid" to print user defined tactics.Gravatar sacerdot2005-05-20
* Extension de Tactic Notation pour permettre d'tendre et de faire rffrence aux...Gravatar herbelin2005-05-17
* Implementation of a new backtracking system, that allow to go backGravatar coq2005-04-20
* Renaming Print Canonical Structure into Print Canonical ProjectionsGravatar herbelin2005-02-18
* Ajout Print Canonical StructuresGravatar herbelin2005-02-12
* Compatibilité ocamlweb pour cible docGravatar herbelin2005-01-21
* Ajout de la syntaxe du reset label: "BackTo n".Gravatar coq2005-01-14
* - Module/Declare Module syntax made more uniform:Gravatar sacerdot2005-01-06
* New command "Print Rewrite HindDb dbname".Gravatar sacerdot2004-11-17
* Ajout 'Locate Module'Gravatar herbelin2004-11-17
* COMMITED BYTECODE COMPILERGravatar barras2004-10-20
* "Print Setoids" command added.Gravatar sacerdot2004-07-23
* Nouvelle en-têteGravatar herbelin2004-07-16
* Réutilisation de VernacSyntacticDefinition pour différencier "Notation id :...Gravatar herbelin2004-01-29
* Reflet dans l'arbre de syntaxe de la difference syntaxique entre 'Variables a...Gravatar herbelin2004-01-13