aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
Commit message (Expand)AuthorAge
* New script dev/tools/change-header to automatically update Coq files headers.Gravatar herbelin2010-06-22
* Fixed bug #2135 (second-order unification was raising cryptic message)Gravatar herbelin2010-06-12
* Added regression tests for bugs + miscellaneous improvementsGravatar herbelin2010-06-12
* Applying François' patch fixing grammar of uniform inheritance condition mes...Gravatar herbelin2010-06-12
* Fixing spelling: pr_coma -> pr_commaGravatar herbelin2010-06-12
* 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
* fixing error message display.Gravatar vgross2010-06-07
* Added support for Ltac-matching terms with variables bound in the patternGravatar herbelin2010-06-06
* Added command "Locate Ltac qid".Gravatar herbelin2010-06-03
* Ide_blob: avoid direct use of Stdpp for compatibility with new camlp4Gravatar letouzey2010-06-03
* Cleanup: remove code specific for ocaml 3.06Gravatar letouzey2010-06-01
* restore handling of lexer errorsGravatar letouzey2010-06-01
* CoqIDE goes multiprocessGravatar vgross2010-05-31
* More indirection.Gravatar vgross2010-05-31
* Introducing strong typing for IDE - toplevel IPCGravatar vgross2010-05-31
* deporting Coq specific code from ide to toplevel.Gravatar vgross2010-05-31
* Modifying startup sequenceGravatar vgross2010-05-31
* New pass on inductive schemesGravatar herbelin2010-05-29
* Add (almost) compatibility with camlp4, without breaking support for camlp5Gravatar letouzey2010-05-19
* Nicer representation of tokens, more independant of camlp*Gravatar letouzey2010-05-19
* static (and shared) camlp4use instead of per-file declarationGravatar letouzey2010-05-19
* Remove compile-command pragmas for emacsGravatar letouzey2010-05-19
* Applicative commutative cuts in Fixpoint guard conditionGravatar pboutill2010-05-18
* - Fixing bug #2308 about Lemma ... withGravatar vsiles2010-05-04
* Fail: a way to check that a command is refused without blocking a scriptGravatar letouzey2010-04-30
* Various minor improvements of comments in mli for ocamldocGravatar letouzey2010-04-29
* Two forgotten $Id$ in last commitGravatar letouzey2010-04-29
* Remove the svn-specific $Id$ annotationsGravatar letouzey2010-04-29
* Move from ocamlweb to ocamdoc to generate mli documentationGravatar pboutill2010-04-29
* Fix bug #2245, incorrect handling of Context in sections inside moduleGravatar msozeau2010-04-27
* Added a new exception for already declared Schemes, Gravatar vsiles2010-04-27
* Here comes the commit, announced long ago, of the new tactic engine.Gravatar aspiwack2010-04-22
* Applying François Garillot's patch (#2261 in bug tracker) for extendedGravatar herbelin2010-04-22
* missing space in error messageGravatar vsiles2010-04-20
* Granting wish #2249 (checking existing lemma name also when in a section).Gravatar herbelin2010-04-09
* Small improvements around coqdoc (including fix for bug #2288)Gravatar herbelin2010-03-30
* Improving error messages in the presence of utf-8 charactersGravatar herbelin2010-03-30
* Several bug-fixes and improvements of coqdocGravatar herbelin2010-03-29
* Fixed bug #2260 (check of resolution of all evars in the declarationGravatar herbelin2010-03-24
* Added automatic expansion on the left of recursive notationsGravatar herbelin2010-03-23
* Fix splitting evars tactics and stop dropping evar constraints whenGravatar msozeau2010-03-15
* No delta-reduction in libtypes anymoreGravatar puech2010-03-11
* Filter out "_subproof" objects from search resultsGravatar puech2010-03-11
* Fix treatment of remaining unification constraints: raise a moreGravatar msozeau2010-03-07
* Fixes in rewrite and a Elimination/Case to Scheme:Gravatar msozeau2010-03-06
* Minor fixes.Gravatar msozeau2010-03-05
* Delineating a API for Coq inside toplevel/vernac.mlGravatar vgross2010-02-12
* New command Declare Reduction <id> := <conv_expr>.Gravatar letouzey2010-01-28
* Variant !F M for functor application that does not honor the Inline declarationsGravatar letouzey2010-01-17