aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened
Commit message (Collapse)AuthorAge
* remove unneeded -emacs flag to coq-prog-argsGravatar Paul Steckler2017-05-01
|
* Merge commit '633ed9c' into v8.6Gravatar Maxime Dénès2016-11-17
|\ | | | | | | Was PR#192: Add test suite files for 4700-4785
| * Add test suite files for 4700-4785Gravatar Jason Gross2016-11-17
| | | | | | | | | | | | | | | | I didn't add any test-cases for timing-based bugs (4707, 4768, 4776, 4777, 4779, 4783), nor CoqIDE bugs (4700, 4751, 4752, 4756), nor bugs about printing (4709, 4711, 4720, 4723, 4734, 4736, 4738, 4741, 4743, 4748, 4749, 4750, 4757, 4758, 4765, 4784). I'm not sure what to do with 4712, 4714, 4732, 4740.
* | Move vector/list compat notations to their relevant filesGravatar Jason Gross2016-09-29
| | | | | | | | | | | | | | Since edb55a94fc5c0473e57f5a61c0c723194c2ff414 landed, compat notations no longer modify the parser in non-compat-mode, so we can do this without breaking Ltac parsing. Also update the related test-suite files.
* | Arguments: cleanup + detect discrepancy rename/implicit (#3753)Gravatar Enrico Tassi2016-09-29
| | | | | | | | | | It seems warnings are not taken into account in output/ tests.
* | Marking bug #3383 as solved.Gravatar Pierre-Marie Pédrot2016-07-18
| |
* | Fix bug #4923: Warning: appcontext is deprecated.Gravatar Pierre-Marie Pédrot2016-07-18
| |
* | Merge branch 'v8.5' into v8.6Gravatar Pierre-Marie Pédrot2016-07-07
|\ \ | |/ |/|
* | Fix test-suite for opened bug #4813.Gravatar Pierre-Marie Pédrot2016-06-15
| |
* | For the record, an example one would like to see working.Gravatar Hugo Herbelin2016-06-12
| |
| * Unbreak singleton list-like notation (-compat 8.4)Gravatar Jason Gross2016-06-09
| | | | | | | | | | | | With this commit, it is possible to write notations so that singleton lists are usable in both 8.4 and 8.5pl1 -compat. Longer lists await the ability to remove notations from the parser.
* | Moving the parsing of the Ltac proof mode to G_ltac.Gravatar Pierre-Marie Pédrot2016-03-19
| |
* | Moving the Tauto tactic to proper Ltac.Gravatar Pierre-Marie Pédrot2016-02-22
| | | | | | | | | | | | This gets rid of brittle code written in ML files through Ltac quotations, and reduces the dependance of Coq to such a feature. This also fixes the particular instance of bug #2800, although the underlying issue is still there.
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-01-13
|\|
| * Fixing #4256 and #4484 (changes in evar-evar resolution made that newGravatar Hugo Herbelin2016-01-12
| | | | | | | | | | | | | | | | evars were created making in turn that evars formerly recognized as pending were not anymore in the list of pending evars). This also fixes the reopening of #3848. See comments on #4484 for details.
* | External tactics and notations now accept any tactic argument.Gravatar Pierre-Marie Pédrot2015-12-30
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This commit has deep consequences in term of tactic evaluation, as it allows to pass any tac_arg to ML and alias tactics rather than mere generic arguments. This makes the evaluation much more uniform, and in particular it removes the special evaluation function for notations. This last point may break some notations out there unluckily. I had to treat in an ad-hoc way the tactic(...) entry of tactic notations because it is actually not interpreted as a generic argument but rather as a proper tactic expression instead. There is for now no syntax to pass any tactic argument to a given ML or notation tactic, but this should come soon. Also fixes bug #3849 en passant.
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-12-17
|\|
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-12-03
|\|
| * Changing syntax "$(tactic)$" into "ltac:(tactic)", as discussed in WG.Gravatar Hugo Herbelin2015-12-02
| |
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-11-15
|\|
| * Now closed.Gravatar Matthieu Sozeau2015-11-11
| |
* | Removing test for bug #3956.Gravatar Pierre-Marie Pédrot2015-10-21
| | | | | | | | | | | | | | It breaks test-suite of trunk since Matthieu's fixes for the soundness of polymorphic universes, and I am unsure of the expected semantics. We should reintroduce it later on when we understand better the issue of simply fix it once and for all.
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-09
|\|
| * Univs: add Strict Universe Declaration option (on by default)Gravatar Matthieu Sozeau2015-10-07
| | | | | | | | | | | | | | | | | | This option disallows "declare at first use" semantics for universe variables (in @{}), forcing the declaration of _all_ universes appearing in a definition when introducing it with syntax Definition/Inductive foo@{i j k} .. The bound universes at the end of a definition/inductive must be exactly those ones, no extras allowed currently. Test-suite files using the old semantics just disable the option.
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-02
|\|
| * Univs: fixed 3685 by side-effect :)Gravatar Matthieu Sozeau2015-10-02
| |
| * Univs: fix test-suite file for HoTT/coq bug #120Gravatar Matthieu Sozeau2015-10-02
| |
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-07-29
|\|
| * Tests for bugs #3509 and #3510.Gravatar Pierre-Marie Pédrot2015-07-28
| |
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-07-18
|\|
| * Remove old test file for #3819 (now fixed).Gravatar Maxime Dénès2015-07-16
| |
* | Temporarily disable test file for #3922.Gravatar Maxime Dénès2015-07-06
| |
* | Fix test file for #4214 which was fixed by Hugo.Gravatar Maxime Dénès2015-06-29
| |
* | Better test case by PMP for #3948.Gravatar Maxime Dénès2015-06-29
| |
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-06-01
|\|
| * 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.
* | Merge v8.5 into trunkGravatar Hugo Herbelin2015-05-15
|\| | | | | | | | | | | | | Conflicts: tactics/eauto.ml4 (merging eauto.ml4 and adapting coq_micromega.ml to new typing.ml API)
* | #3953 now closed.Gravatar Hugo Herbelin2015-05-14
| |
| * 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.
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-05-05
|\|
| * 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.
* | Merge branch 'v8.5' into trunkGravatar Enrico Tassi2015-03-30
|\|
| * Updating test-suite (see previous commit).Gravatar Hugo Herbelin2015-03-24
| |
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-03-11
|\|
| * 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
| * Test for bug #2951.Gravatar Pierre-Marie Pédrot2015-03-08
| |
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-03-04
|\|
| * Fix test-suite file, this is open.Gravatar Matthieu Sozeau2015-03-03
| |