aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
Commit message (Collapse)AuthorAge
* admit: replaced by give_up + Admitted (no proof_admitted : False, close #4032)Gravatar Enrico Tassi2015-03-11
| | | | | | | | | | | | | | | - no more inconsistent Axiom in the Prelude - STM can now process Admitted proofs asynchronously - the quick chain can stock "Admitted" jobs in .vio files - the vio2vo step checks the jobs but does not stock the result in the opaque tables (they have no slot) - Admitted emits a warning if the proof is complete - Admitted uses the (partial) proof term to infer section variables used (if not given with Proof using), like for Qed - test-suite: extra line Require TestSuite.admit to each file making use of admit - test-suite/_CoqProject: to pass to CoqIDE and PG the right -Q flag to find TestSuite.admit
* Do not display the status of monomorphic constants unless in ↵Gravatar Guillaume Melquiond2015-03-09
| | | | universe-polymorphism mode.
* Test for bug #2951.Gravatar Pierre-Marie Pédrot2015-03-08
|
* Test for #4035 (dependent destruction from Ltac).Gravatar Hugo Herbelin2015-03-07
|
* Fix testsuite with respect to the new formatting of Fail messages.Gravatar Guillaume Melquiond2015-03-05
|
* Fix test-suite file, this is open.Gravatar Matthieu Sozeau2015-03-03
|
* Fix bug #3732: firstorder was using detyping to build existentialGravatar Matthieu Sozeau2015-03-03
| | | | | | instances and forgeting about the evars and universes that could appear there... dirty hack gone, using the evar map properly and avoiding needless constructions/deconstructions of terms.
* Add missing test-suite files and update gitignore.Gravatar Matthieu Sozeau2015-03-03
|
* Add a test-suite file ensuring coinductives with primitive projectionsGravatar Matthieu Sozeau2015-03-03
| | | | | do not enjoy eta-conversion and do not allow the usual failure of subject reduction in presence of dependent pattern-matching.
* Fix test-suite file, this is currently a wontfix, but keep theGravatar Matthieu Sozeau2015-03-03
| | | | test-suite file for when we move to a better implementation.
* Fix bug #4103: forgot to allow unfolding projections of cofixpoints likeGravatar Matthieu Sozeau2015-03-03
| | | | cases, in some cases.
* Fix bug #4101, noccur_evar's expand_projection can legitimately failGravatar Matthieu Sozeau2015-03-03
| | | | when called from w_unify, so we protect it.
* Fix bug #4097.Gravatar Matthieu Sozeau2015-03-02
|
* Adding a test for bug #3612.Gravatar Pierre-Marie Pédrot2015-02-27
|
* Test for bug #3249.Gravatar Pierre-Marie Pédrot2015-02-27
|
* Fix test for #3467, I had moved it in a dumb way.Gravatar Maxime Dénès2015-02-27
|
* Add support so that the type of a match in an inductive type with let-inGravatar Hugo Herbelin2015-02-27
| | | | | | | | | is reduced as if without let-in, when applied to arguments. This allows e.g. to have a head-betazeta-reduced goal in the following example. Inductive Foo : let X := Set in X := I : Foo. Definition foo (x : Foo) : x = x. destruct x. (* or case x, etc. *)
* Fixing first part of bug #3210 (inference of pattern-matching returnGravatar Hugo Herbelin2015-02-27
| | | | clause in the presence of let-ins in the arity of inductive type).
* Fix test for #3848, still open.Gravatar Maxime Dénès2015-02-27
|
* Moving test for #3467 to closed after PMP's fix.Gravatar Maxime Dénès2015-02-27
|
* Fix test-suite files for bugs #2456 and #3593, still open.Gravatar Maxime Dénès2015-02-27
|
* Add test-suite file for #3649.Gravatar Maxime Dénès2015-02-27
|
* Moving tests for #2456 and #3593 to "opened" until they're fixed.Gravatar Maxime Dénès2015-02-27
|
* Made test for #3392 rely less on unification.Gravatar Maxime Dénès2015-02-27
|
* Moving test of #3848 to "opened".Gravatar Maxime Dénès2015-02-27
|
* Test for #2602, which seems now fixed.Gravatar Maxime Dénès2015-02-26
|
* Test for bug #3298.Gravatar Pierre-Marie Pédrot2015-02-26
|
* Fixing complexity tests for #4076.Gravatar Maxime Dénès2015-02-26
|
* Revert "Fixing bug #4035 (support for dependent destruction within ltac code)."Gravatar Maxime Dénès2015-02-26
| | | | | | | | | This reverts commit 4e6c9891140932f452bb5ac8960d597b0b5fde1d, which was breaking compatibility because one could no longer use names of foralls in the goal without introducting them. Probably not good style, but it did break many existing developments including CompCert. Closes #4093 but reopens #4035.
* Moving test for bug #3681 as closed.Gravatar Pierre-Marie Pédrot2015-02-26
|
* Another test for a variant of complexity problem #4076 (thanks to A. Mortberg).Gravatar Hugo Herbelin2015-02-25
|
* Univs: Fix Check calling the kernel to retype in the wrong environment.Gravatar Matthieu Sozeau2015-02-24
| | | | Fixes bug #4089.
* Compensating 6fd763431 on postponing subtyping evar-evar problems.Gravatar Hugo Herbelin2015-02-23
| | | | | | | Pushing pending problems had the side-effect of later solving them in the opposite order as they arrived, resulting on different complexity (see e.g. #4076). We now take care of pushing them in reverse order so that they are treated in the same order.
* Fix some typos in comments.Gravatar Guillaume Melquiond2015-02-23
|
* Test for #3953 (subst in evar instances).Gravatar Hugo Herbelin2015-02-23
|
* Fixing rewrite/subst when the subterm to rewrite is argument of an Evar.Gravatar Hugo Herbelin2015-02-23
| | | | | | | | | | | | This was broken by the attempt to use the same algorithm for rewriting closed subterms than for rewriting subterms with evars: the algorithm to find subterms (w_unify_to_subterm) did not go through evars. But what to do when looking say, for a pattern "S ?n" in a goal "S ?x[a:=S ?y]"? Should we unify ?x[a:=S ?y] with ?n or consider ?x as rigid and look in the instance? If we adopt the first approach, then, what to do when looking for "S ?n" in a goal "?x[a:=S ?y]"? Failing? Looking in the instance? Is it normal that an evar behaves as a rigid constant when it cannot be unified with the pattern?
* Fixing occur-check which was too strong in unification.ml.Gravatar Hugo Herbelin2015-02-23
|
* Fixing test #2830.Gravatar Pierre-Marie Pédrot2015-02-23
|
* Fixing test for bug #3071.Gravatar Pierre-Marie Pédrot2015-02-23
|
* Moving test for bug #3071.Gravatar Pierre-Marie Pédrot2015-02-21
|
* Test for bug #4078.Gravatar Pierre-Marie Pédrot2015-02-21
|
* A fix for #3993 (not fully applied term to destruct when eqn is given).Gravatar Hugo Herbelin2015-02-20
|
* Fix bug #3938Gravatar Matthieu Sozeau2015-02-18
|
* Remove some dead code and add test-suite file.Gravatar Matthieu Sozeau2015-02-16
|
* Add test-suite file for #3960.Gravatar Matthieu Sozeau2015-02-16
|
* Test for bug #3922.Gravatar Pierre-Marie Pédrot2015-02-16
|
* Fixing bug #4035 (support for dependent destruction within ltac code).Gravatar Hugo Herbelin2015-02-16
|
* Test for #2946 (trunk bug with let's in unification).Gravatar Hugo Herbelin2015-02-16
|
* Fixing test for bug #3944.Gravatar Pierre-Marie Pédrot2015-02-16
|
* Test for bug #3944.Gravatar Pierre-Marie Pédrot2015-02-16
|