aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
Commit message (Collapse)AuthorAge
* Fix bug #4254 with the help of J.H. JourdanGravatar Matthieu Sozeau2015-06-26
| | | | | | | | | | | | | | | 1) We now _assign_ the smallest possible arities to mutual inductive types and eventually add leq constraints on the user given arities. Remove useless limitation on instantiating algebraic universe variables with their least upper bound if they have upper constraints as well. 2) Do not remove non-recursive variables when computing minimal levels of inductives. 3) Avoid modifying user-given arities if not necessary to compute the minimal level of an inductive. 4) We correctly solve the recursive equations taking into account the user-declared level.
* Fix test-suite after 1343b69221ce3eeb3154732e73bbdc0044b224a8.Gravatar Maxime Dénès2015-06-24
|
* Fixing incompatibility introduced with simpl in commit 364decf59c1 (orGravatar Hugo Herbelin2015-06-23
| | | | | | | | | | | maybe ca71714). Goal 2=2+2. match goal with |- (_ = ?c) => simpl c end. was working in 8.4 but was failing in 8.5beta2. Note: Changes in tacintern.ml are otherwise purely cosmetic.
* Add test-suite file for bug #3446.Gravatar Matthieu Sozeau2015-06-11
|
* STM: states coming from workers have no proof terminators (Close #4246)Gravatar Enrico Tassi2015-06-09
| | | | Hence we reuse the ones in master.
* STM: silly mistake in jumping back to an old state (Close #4249)Gravatar Enrico Tassi2015-06-09
|
* Adding a test for bug #4057.Gravatar Pierre-Marie Pédrot2015-06-02
|
* Flag -test-mode intended to be used for ad-hoc prints in test-suiteGravatar Enrico Tassi2015-05-29
| | | | | | | Of course there is an exception to the previous commit. Fail used to print even if silenced but loading a vernac file. This behavior is useful only in tests, hence this flag.
* STM: preserve branch name on edit (Close: #4245, #4246)Gravatar Enrico Tassi2015-05-28
|
* Test for 4159Gravatar Enrico Tassi2015-05-28
|
* Test for bug #4116.Gravatar Pierre-Marie Pédrot2015-05-19
|
* Removing test for opened bugs that were already present in the closed ↵Gravatar Pierre-Marie Pédrot2015-05-18
| | | | test-suite.
* Tentative fix for #3461: Anomaly: Uncaught exception ↵Gravatar Pierre-Marie Pédrot2015-05-18
| | | | | | Pretype_errors.PretypeError. Instad of trying to print the exception, we raise it in the tactic monad.
* Removing option -no-native-compiler from test #3539 since this option is nowGravatar Hugo Herbelin2015-05-15
| | | | negated into -native-compiler.
* Fixing bug #4216:Gravatar Pierre-Marie Pédrot2015-05-13
| | | | | | Internal error: Anomaly: Uncaught exception Not_found. Please report. An evarmap was lost because of an unsound typing primitive.
* Better fixing #4198 such that the term to match is looked for beforeGravatar Hugo Herbelin2015-05-13
| | | | | | | the predicate, thus respecting the visual left-to-right top-down order (see a45bd5981092). This fixes CFGV.
* Extraction: fix the detection of the "polyprop" situationGravatar Pierre Letouzey2015-05-12
| | | | | | | | The ~polyprop argument wasn't propagated properly anymore, leading the extraction to try to operate on situations it cannot handle (yet). Cf Table.error_singleton_become_prop for more details. Regression test added.
* Test for bug #4234.Gravatar Pierre-Marie Pédrot2015-05-12
|
* Test for bug #4232.Gravatar Pierre-Marie Pédrot2015-05-11
|
* Adjusting test-suite after 5cbc018fe9347 (subst as in 8.4 by default).Gravatar Hugo Herbelin2015-05-09
|
* Adding a flag "Set Regular Subst Tactic" off by default in v8.5 forGravatar Hugo Herbelin2015-05-09
| | | | preserving compatibility of subst after #4214 being solved.
* Fixing treatment of recursive equations damaged by 857e82b2ca0d1.Gravatar Hugo Herbelin2015-05-06
| | | | | | Improving treatment of recursive equations compared to 8.4 (see test-suite). Experimenting not to unfold local defs ever in subst. (+ Slight simplification in checking reflexive equalities only once).
* Fixing computation of implicit arguments by position in fixpoints (#4217).Gravatar Hugo Herbelin2015-05-01
|
* Giving to "subst" a more natural semantic (fixing #4214) by using allGravatar Hugo Herbelin2015-05-01
| | | | | | | | | | | | | | | | | | | | | equalities in configurations like x=y x=z === P(x,y,z) where it now produces === P(z,z,z) In particular (equations are processed from most ancient to most recent). Thanks to this, a "repeat subst" can just be a "subst" in List.v. Incidentally: moved a nf_enter to enter in subst_one, since the latter is normally called from other tactics having normalized evars.
* Tactical `progress` compares term up to potentially equalisable universes.Gravatar Arnaud Spiwack2015-04-22
| | | | | Followup of: f7b29094fe7cc13ea475447bd30d9a8b942f0fef . In particular, re-closes #3593. As a side effect, fixes an undiscovered bug of the `eq_constr` tactic which didn't consider terms up to evar instantiation.
* Test for #4198 (appcontext in return clause of match).Gravatar Hugo Herbelin2015-04-22
|
* Fixing #3376 and #4191 (wrong index of maximally-inserted implicit argumentGravatar Hugo Herbelin2015-04-21
| | | | in the presence of let-ins).
* Extra fix to 934761875 and f4ee7ee31e4 on optimizing Import of severalGravatar Hugo Herbelin2015-04-17
| | | | libraries at once (see #4193).
* Test for bug #4190.Gravatar Pierre-Marie Pédrot2015-04-16
|
* Test for bug #3199.Gravatar Pierre-Marie Pédrot2015-04-10
|
* Better test-suite files, removing reliance on admit.Gravatar Matthieu Sozeau2015-04-09
|
* Fix declarations of instances to perform restriction of universeGravatar Matthieu Sozeau2015-04-09
| | | | instances as definitions and lemmas do (fixes bug# 4121).
* Add test-suite file for bug #4120.Gravatar Matthieu Sozeau2015-04-09
|
* Test for bug #3815.Gravatar Pierre-Marie Pédrot2015-04-06
|
* Fixing test-suite.Gravatar Pierre-Marie Pédrot2015-04-01
|
* Fixing test-suite.Gravatar Pierre-Marie Pédrot2015-03-31
|
* camlp4: grep away warnings in output/* testsGravatar Enrico Tassi2015-03-30
|
* Adding test for bug #4165.Gravatar Pierre-Marie Pédrot2015-03-29
|
* Fully fixing bug #3491 (anomaly when building _rect scheme in theGravatar Hugo Herbelin2015-03-25
| | | | | | | | | | | | presence of let-ins and recursively non-uniform parameters). The bug was in the List.chop of Inductiveops.get_arity which was wrong in the presence of let-ins and recursively non-uniform parameters. The bug #3491 showed up because, in addition to have let-ins, it was wrongly detected as having recursively non-uniform parameters. Also added some comments in declarations.mli.
* Another example about the consequence of a wrong computation of theGravatar Hugo Herbelin2015-03-25
| | | | | | | | number of recursively uniform parameters in the presence of let-ins. In practice, more recursively non-uniform parameters were assumed and this was used especially for checking positivity of nested types, leading to refusing more nested types than necessary (see Inductive.v).
* Updating test-suite (see previous commit).Gravatar Hugo Herbelin2015-03-24
|
* Fixing computation of non-recursively uniform arguments in theGravatar Hugo Herbelin2015-03-24
| | | | presence of let-ins. This fixes #3491.
* Fixing wrong rel_context in checking positivity condition.Gravatar Hugo Herbelin2015-03-24
| | | | | | | | | | Parameters were missing in the context, apparently without negative effects because the context was used only for whd normalization of types, while reduction (in closure.ml) was resistant to unbound rels. See however next commit for an indirect effect on the wrong computation of non recursively uniform parameters producing an anomaly when computing _rect schemas.
* Qed export -> Qed exportingGravatar Enrico Tassi2015-03-22
|
* Add some tests for tryifGravatar Jason Gross2015-03-13
| | | | + adjusting for the removal of `admit` by Arnaud Spiwack.
* Fix regression in HoTT_coq_014.vGravatar Enrico Tassi2015-03-11
| | | | | Admitted was not using the partial proof to infer discharged variables. Now it does. The fix makes no sense, but restore the old behavior.
* 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
|