aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/command.mli
Commit message (Expand)AuthorAge
* get rid of closures in global/proof stateGravatar gareuselesinge2013-08-08
* State Transaction MachineGravatar gareuselesinge2013-08-08
* Use the Hook module here and there.Gravatar ppedrot2013-05-12
* A uniformization step around understand_* and interp_* functions.Gravatar herbelin2013-05-09
* Declaration of multiple hypotheses or parameters now share typingGravatar herbelin2013-05-08
* Fix bug# 2994, 2971 about better error messages.Gravatar msozeau2013-03-22
* Modules and ppvernac, sequel of Enrico's commit 16261Gravatar letouzey2013-03-13
* Allowing (Co)Fixpoint to be defined local and Let-style.Gravatar ppedrot2013-03-11
* Modulification of nameGravatar ppedrot2012-12-18
* Modulification of identifierGravatar ppedrot2012-12-14
* Assumption commands are now displayed as unsafe in Coqide.Gravatar aspiwack2012-08-24
* Updating headers.Gravatar herbelin2012-08-08
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar letouzey2012-05-29
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar letouzey2012-05-29
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14
* Integrated obligations/eterm and program well-founded fixpoint building to to...Gravatar msozeau2012-03-14
* Noise for nothingGravatar pboutill2012-03-02
* Revert "Add [Polymorphic] flag for defs"Gravatar msozeau2011-04-13
* Add [Polymorphic] flag for defsGravatar msozeau2011-04-13
* Annotations at functor applications:Gravatar letouzey2011-02-11
* More comments and less doublons in some mliGravatar pboutill2011-02-10
* A fine-grain control of inlining at functor application via priority levelsGravatar letouzey2011-01-31
* Remove the "Boxed" syntaxes and the const_entry_boxed fieldGravatar letouzey2011-01-28
* Updated all headers for 8.3 and trunkGravatar herbelin2010-07-24
* Amelioration dans FunctionGravatar jforest2010-07-16
* change the flag "internal" in declare/ind_tables from bool toGravatar vsiles2010-06-29
* New script dev/tools/change-header to automatically update Coq files headers.Gravatar herbelin2010-06-22
* Automatic introduction of names given before ":" in Lemma's andGravatar herbelin2010-06-09
* Fix treatment of {struct x} annotations in presence of generalizedGravatar msozeau2010-06-08
* Various minor improvements of comments in mli for ocamldocGravatar letouzey2010-04-29
* Remove the svn-specific $Id$ annotationsGravatar letouzey2010-04-29
* Move from ocamlweb to ocamdoc to generate mli documentationGravatar pboutill2010-04-29
* Added support for definition of fixpoints using tactics.Gravatar herbelin2009-11-27
* Added support for multiple where-clauses in Inductive and co (see wish #2163).Gravatar herbelin2009-11-11
* Restructuration of command.ml + generic infrastructure for inductive schemesGravatar herbelin2009-11-08
* Delete trailing whitespaces in all *.{v,ml*} filesGravatar glondu2009-09-17
* Backtrack on the forced discharge of type class variables introducedGravatar msozeau2009-09-14
* Fix implicit args code so that declarations are added for allGravatar msozeau2009-05-27
* Fix to my last notation patch: now fixpoint are correctly handled Gravatar vsiles2009-05-13
* Fixed bugs #2001 (search_guard was overwriting the guard index givenGravatar herbelin2009-01-04
* More factorization of inductive/record and typeclasses: move classGravatar msozeau2008-11-09
* Nouvelle syntaxe pour écrire des records (co)inductifs :Gravatar aspiwack2008-11-05
* Add enough information to correctly globalize recursive calls in inductive andGravatar msozeau2008-09-11
* Fix bug #1913, checking for unresolved evars which aren't obligations.Gravatar msozeau2008-07-24
* Improvements on coqdoc by adding more information into .globGravatar msozeau2008-05-30
* Postpone the search for the recursive argument index from the user givenGravatar msozeau2008-05-06
* Ajout de "Theorem id1 : t1 ... with idn : tn" pour partager la preuveGravatar herbelin2008-04-25
* Add the ability to specify the implicit status of section variables andGravatar msozeau2008-04-02
* Ajout d'abbréviations/notations paramétriquesGravatar herbelin2008-03-30