aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
Commit message (Expand)AuthorAge
* A slightly more efficient test of well-typedness of restriction ofGravatar herbelin2013-02-21
* Added propagation of evars unification failure reasons for betterGravatar herbelin2013-02-17
* Revised the Ltac trace mechanism so that trace breaking due toGravatar herbelin2013-02-17
* Fixed bug #2981 (anomaly NotASort in Retyping due to collision betweenGravatar herbelin2013-02-05
* Fixed #2970 (made that remember's eqn name is interpretable as an ltac var).Gravatar herbelin2013-01-29
* Added a file for testing regression of bug #2955 (anomaly in simpl inGravatar herbelin2013-01-29
* Fixing bug #2969 (admit failing after Grab Existential Variables dueGravatar herbelin2013-01-29
* Fixed bug #2966 (de Bruijn error in computation of heads for coercions).Gravatar herbelin2013-01-28
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* Fixing one part of #2830 (anomaly "defined twice" due to nested calls toGravatar herbelin2013-01-28
* Fix bug 2958: Inductive deep in in clause are impossibleGravatar pboutill2013-01-21
* Last test-suite not in Symmetric Patterns syntaxGravatar pboutill2013-01-21
* Unset Asymmetric PatternsGravatar pboutill2013-01-18
* Fixing parsing of specific primitive tokens used as notations for patternsGravatar herbelin2012-12-18
* Taking into account the possibility of having a type of type which isGravatar herbelin2012-12-18
* Fixed a little inefficiency of "set/destruct" over a pattern. NowGravatar herbelin2012-12-18
* Backtrack on activating scopes with type casts (was r15978).Gravatar herbelin2012-12-04
* Revised the strategy for automatic insertion of spaces when printingGravatar herbelin2012-12-04
* Evarconv: Fix #2936 + commentsGravatar pboutill2012-11-28
* Fixed bug #2930: folded let-in's were hiding a violation to the occurGravatar herbelin2012-11-25
* Fixing test-suite: Scope.vGravatar ppedrot2012-11-21
* Hurkens' paradox on Type (r15973 and r15977) needs two (non-Set)Gravatar herbelin2012-11-18
* Update output/Search.out after hint-related extra defs in PeanoGravatar letouzey2012-11-17
* Taking into account the type of a definition (if it exists), and theGravatar herbelin2012-11-17
* Fix test-suite output/* in benchGravatar pboutill2012-10-17
* test-suite: fix grep rule for output testsGravatar pboutill2012-09-04
* test-suite uses coqtop instead of coqtop.byteGravatar pboutill2012-09-04
* In the output tests, ignore dynlink messagesGravatar letouzey2012-08-24
* test-suite: Local Tactic Notation is now legal since r15731Gravatar letouzey2012-08-23
* No more coqtop.opt, produce directly a coqtop binaryGravatar letouzey2012-08-23
* Unification in Evar_conv uses an abstract machine stateGravatar pboutill2012-08-09
* Updating headers.Gravatar herbelin2012-08-08
* Fixing #2836 (materialize_evar might refine as a side effect theGravatar herbelin2012-07-29
* Fixing bug #2835 (the rationale for printing notations was notGravatar herbelin2012-07-21
* Improving management of notations with binders (see #2708 where aGravatar herbelin2012-07-21
* Restore test file induct.v where the "in |- *" is mandatoryGravatar letouzey2012-07-10
* Continuing r15459: it helps testing occur-check early in someGravatar herbelin2012-07-06
* Minor fixes in the test-suite after my recent commitsGravatar letouzey2012-07-06
* Legacy Ring and Legacy Field migrated to contribsGravatar letouzey2012-07-05
* Kills the useless tactic annotations "in |- *"Gravatar letouzey2012-07-05
* Open Local Scope ---> Local Open Scope, same with Notation and aliiGravatar letouzey2012-07-05
* ZArith + other : favor the use of modern names instead of compat notationsGravatar letouzey2012-07-05
* Fixing bug #2817 (occur check was not done up to instantiation ofGravatar herbelin2012-06-20
* Fixing bug #2809 (anomaly when printing a module with notations due toGravatar herbelin2012-06-20
* Proof using: nested sections bugfixGravatar gareuselesinge2012-06-18
* Constrextern is allow to use partially applied notationsGravatar pboutill2012-06-14
* Fixing test-suite after last storm in Pp.Gravatar pboutill2012-06-12
* Changed encoding from ISO-8859-1 to UTF-8 for some remaining gallina files.Gravatar ppedrot2012-06-12
* Notations are back in the "in" clause of pattern matching.Gravatar pboutill2012-05-15
* Implicit arguments of Definition are taken from the type when given by the user.Gravatar pboutill2012-04-27