aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
...
* Fix typeclass resolution error message which included goal evars (bug #2620).Gravatar msozeau2012-01-23
* Fix for Program Instance not separately checking the resolution of evars of t...Gravatar msozeau2012-01-23
* Another quick hack that works this time, to handle printing of locality in Pr...Gravatar ppedrot2012-01-23
* Deleted the only use of BeginSubProof from the standard library.Gravatar ppedrot2012-01-23
* Removed a seemingly unused argument in Require of modules, introduced 10 year...Gravatar ppedrot2012-01-23
* Fixed pretty-printing of Opaque, Transparent and Strategy locality flags.Gravatar ppedrot2012-01-23
* Bug 739: forbid dumpglob while using Coqtop in interactive modeGravatar pboutill2012-01-23
* Coqtop and coqc: cleaning description of options in RefMan and manpages.Gravatar pboutill2012-01-21
* Added documentation for "r foo" in Ltac debugger.Gravatar herbelin2012-01-20
* Added documentation for "Set Parsing Explicit" + fixed mistakenlyGravatar herbelin2012-01-20
* Breakpoints in Ltac debugger: new command "r foo" to jump to the nextGravatar herbelin2012-01-20
* Added new command "Set Parsing Explicit" for deactivating parsing (andGravatar herbelin2012-01-20
* Notations with binders: Accepting using notations for functional termsGravatar herbelin2012-01-20
* Reverted previous commit, which broke library compilation.Gravatar ppedrot2012-01-20
* This is a quick hack to permit the parsing of the locality flag in the Progra...Gravatar ppedrot2012-01-20
* Fix printing of classesGravatar msozeau2012-01-20
* Fix typeclass constraint grammar rule to allow `{_ : Reflexive A R}.Gravatar msozeau2012-01-19
* Added the btauto tactic to the documentation.Gravatar ppedrot2012-01-19
* Pretty printing of generalized binderGravatar pboutill2012-01-19
* Boolean Option Patterns CompatibilityGravatar pboutill2012-01-19
* No more use of tauto in Init/Gravatar pboutill2012-01-19
* Fixed the pretty-printing of the Program plugin.Gravatar ppedrot2012-01-17
* Makefile: fix make distclean w.r.t. test-suiteGravatar letouzey2012-01-17
* MSetAVL: better implementation of filter suggested by X. LeroyGravatar letouzey2012-01-17
* Some fix in beautify pretty-printerGravatar pboutill2012-01-17
* Parameters in pattern first step.Gravatar pboutill2012-01-16
* Inductiveops.nb_*{,_env} cleaningGravatar pboutill2012-01-16
* Bug 2679: Do not try to install cmxs with -byte-onlyGravatar pboutill2012-01-16
* Bug 2676: ./configure --prefix shoudn't ask for a config directory.Gravatar pboutill2012-01-16
* make mli-doc fixGravatar pboutill2012-01-16
* coq_micromega.ml: fix order of recursive calls to rconstantGravatar glondu2012-01-14
* Add distclean back to test-suite/MakefileGravatar glondu2012-01-14
* More newlines in debugging output of psatzlGravatar glondu2012-01-14
* Added a Btauto plugin, that solves boolean tautologies.Gravatar ppedrot2012-01-13
* Added the decidability of (<=) on nat.Gravatar ppedrot2012-01-13
* Fix typoGravatar glondu2012-01-12
* Fix printing of instances, generalized arguments.Gravatar msozeau2012-01-10
* Fix typoGravatar glondu2012-01-07
* Fixed the itarget of the previous commit...Gravatar ppedrot2012-01-06
* Added a typeclass-based system to reason on decidable propositions.Gravatar ppedrot2012-01-06
* Forbids (as it has always been the behaviour) to have two different openGravatar aspiwack2012-01-06
* Fixes bug #2654 (tactic instantiate failing to update existential variables).Gravatar aspiwack2012-01-06
* Backtracking on r14876 (fix for bug #2267): extra scopes might beGravatar herbelin2012-01-05
* Fixing Arguments Scope bug when too many scopes are given (bug #2667).Gravatar herbelin2012-01-04
* Type inference unification: fixed a 8.4 bug in the presence of unificationGravatar herbelin2012-01-04
* Makefile.doc: attempt to solve race condition for creating doc/refman/html.Gravatar herbelin2012-01-03
* Bug 2669 and more: make full-stdlibGravatar pboutill2011-12-27
* Coqdoc: Fixing missing newline when using "Proof term."Gravatar herbelin2011-12-26
* Reference Manual: misc fixes (spelling, index, updating pre-8.0 syntax).Gravatar herbelin2011-12-26
* update CHANGES w.r.t. simplGravatar gareuselesinge2011-12-26