aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Compat
Commit message (Collapse)AuthorAge
* Add empty compat file for Coq 8.8Gravatar Jason Gross2018-03-07
| | | | This closes #6598
* Merge PR #6855: Update headers following #6543.Gravatar Maxime Dénès2018-03-05
|\
* | Remove 8.5 compatibility support.Gravatar Théo Zimmermann2018-03-02
| |
| * Update headers following #6543.Gravatar Théo Zimmermann2018-02-27
|/
* Fix (partial) #4878: option to stop autodeclaring axiom as instance.Gravatar Gaëtan Gilbert2017-11-28
|
* Compat/Coq87.v : Unset Omega UseLocalDefs (see PR #768)Gravatar Pierre Letouzey2017-10-07
|
* Adding a V8.7 compatibility version number.Gravatar Hugo Herbelin2017-07-21
|
* Bump year in headers.Gravatar Pierre-Marie Pédrot2017-07-04
|
* Put plugin exports in the right compatibility fileGravatar Jason Gross2017-06-22
| | | | | | | | This closes [bug #5607](https://coq.inria.fr/bugs/show_bug.cgi?id=5607). PR #220 put the exports in the wrong compat files, presumably because it was originally targeted to version 8.6, and this wasn't updated when it was retargeted to version 8.7.
* Merge PR#375: DeprecationGravatar Maxime Dénès2017-06-15
|\
* | Prelude : no more autoload of plugins extraction and recdefGravatar Pierre Letouzey2017-06-14
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | The user now has to manually load them, respectively via: Require Extraction Require Import FunInd The "Import" in the case of FunInd is to ensure that the tactics functional induction and functional inversion are indeed in scope. Note that the Recdef.v file is still there as well (it contains complements used when doing Function with measures), and it also triggers a load of FunInd.v. This change is correctly documented in the refman, and the test-suite has been adapted.
| * Remove support for Coq 8.4.Gravatar Guillaume Melquiond2017-06-14
|/
* drop vo.itarget files and compute the corresponding the corresponding values ↵Gravatar Matej Kosik2017-06-01
| | | | automatically instead
* Merge commit 'e6edb33' into v8.6Gravatar Maxime Dénès2016-11-07
|\ | | | | | | Was PR#331: Solve_constraints and Set Use Unification Heuristics
| * More explicit name for status of unification constraints.Gravatar Maxime Dénès2016-11-07
| |
* | Silence option deprecation warnings in the compat fileGravatar Jason Gross2016-11-04
| | | | | | | | Some options are expected to be deprecated
| * Add Unset Use Unif Heuristics in Compat/Coq85Gravatar Matthieu Sozeau2016-10-22
|/
* Fix previous commit.Gravatar Pierre-Marie Pédrot2016-10-17
| | | | I've messed up with parts of the compatibility files I had to commit.
* Merge PR #300 into v8.6Gravatar Pierre-Marie Pédrot2016-10-17
|\
* | Clean up type classes flags and update compat file.Gravatar Maxime Dénès2016-10-05
| |
| * 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.
* Remove spaces from around list notationsGravatar Jason Gross2016-09-26
|
* Unbreak Ltac [ | .. | ] notation in -compat 8.5Gravatar Jason Gross2016-09-26
| | | | | | Importing VectorNotations breaks `; []`. So we make sure it's not imported by defualt. Some files might be required to `Import VectorDef.VectorNotations` rather than just `Import VectorNotations`.
* Fix bug #4785 (use [ ] for vector nil)Gravatar Jason Gross2016-09-26
| | | | | Also delimit vector_scope with vector, so that people can write %vector without having to delimit it themselves.
* Refolding: disable in 8.4 compat file, documentGravatar Matthieu Sozeau2016-09-12
|
* no-refold patchGravatar Paul Steckler2016-09-09
| | | | | | Add a boolean for refolding during reduction, and an option that is off by default in 8.6, to turn refolding on in all reduction functions, as in 8.5.
* Merge branch 'v8.5' into v8.6Gravatar Pierre-Marie Pédrot2016-09-02
|\
| * Fix bug #5043: [Admitted] lemmas pick up section variables.Gravatar Pierre-Marie Pédrot2016-08-31
| | | | | | | | | | | | We add a flag Keep Admitted Variables that allows to recover the legacy v8.4 behaviour of admitted lemmas. The statement of such lemmas did not depend on the current context variables.
* | Merge branch 'v8.5' into v8.6Gravatar Pierre-Marie Pédrot2016-07-07
|\|
* | Fix #4793: Coq 8.6 should accept -compat 8.6Gravatar Maxime Dénès2016-07-06
| | | | | | | | We also add a Coq86.v compat file.
| * Compat84: Don't mess with stdlib modulesGravatar Jason Gross2016-07-05
| | | | | | | | | | | | | | | | | | We don't actually need to, unless we want to support the (presumably uncommon) use-case of someone using [Import VectorNotations] to override their local notation for things in vector_scope. Additionally, we now maintain the behavior that [Import VectorNotations] opens vector_scope.
* | Add Unset Shrink Abstract/Obligations in Coq85Gravatar Matthieu Sozeau2016-06-27
| | | | | | | | For compatibility with 8.5.
* | Giving a more natural semantics to injection by default.Gravatar Hugo Herbelin2016-06-18
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | There were three versions of injection: 1. "injection term" without "as" clause: was leaving hypotheses on the goal in reverse order 2. "injection term as ipat", first version: was introduction hypotheses using ipat in reverse order without checking that the number of ipat was the size of the injection (activated with "Unset Injection L2R Pattern Order") 3. "injection term as ipat", second version: was introduction hypotheses using ipat in left-to-right order checking that the number of ipat was the size of the injection and clearing the injecting term by default if an hypothesis (activated with "Set Injection L2R Pattern Order", default one from 8.5) There is now: 4. "injection term" without "as" clause, new version: introducing the components of the injection in the context in left-to-right order using default intro-patterns "?" and clearing the injecting term by default if an hypothesis (activated with "Set Structural Injection") The new versions 3. and 4. are the "expected" ones in the sense that they have the following good properties: - introduction in the context is in the natural left-to-right order - "injection" behaves the same with and without "as", always introducing the hypotheses in the goal what corresponds to the natural expectation as the changes I made in the proof scripts for adaptation confirm - clear the "injection" hypothesis when an hypothesis which is the natural expectation as the changes I made in the proof scripts for adaptation confirm The compatibility can be preserved by "Unset Structural Injection" or by calling "simple injection". The flag is currently off.
| * 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.
* | Relying instead on the Coq85 inclusion!Gravatar Hugo Herbelin2016-06-06
| |
* | Mode "Bracketing Last Introduction Pattern" is on for 8.4Gravatar Hugo Herbelin2016-06-06
| | | | | | | | and global for 8.4 and 8.5.
* | Mode "Regular Subst Tactic" is on in 8.6.Gravatar Hugo Herbelin2016-06-06
| |
* | Merge remote-tracking branch 'github/pr/118' into trunkGravatar Maxime Dénès2016-06-06
|\ \
* \ \ Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-05-20
|\ \ \ | | |/ | |/|
| * | Removing unexcepted activation of option "Regular Subst Tactic", sinceGravatar Hugo Herbelin2016-05-14
| | | | | | | | | | | | there is actually no change in default subst between 8.4 and 8.5.
* | | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-05-04
|\| |
| * | Merge branch 'move-compat-notations' of https://github.com/JasonGross/coq ↵Gravatar Pierre Letouzey2016-05-04
| |\ \ | | | | | | | | | | | | into v8.5
* | | | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-04-09
|\| | |
| * | | Added compatibility coercions from Specif.v which were present in Coq 8.4.Gravatar Hugo Herbelin2016-04-08
| | | |
| * | | Add -compat 8.4 econstructor tactics, and testsGravatar Jason Gross2016-04-05
| | | | | | | | | | | | | | | | | | | | Passing `-compat 8.4` now allows the use of `econstructor (tac)`, as in 8.4.
| * | | Fix bug #4656Gravatar Jason Gross2016-04-05
| | | | | | | | | | | | | | | | | | | | I introduced this bug in 4c078b0362542908eb2fe1d63f0d867b339953fd; Coq.Init.Notations.constructor does not take any arguments.
| * | | Update Coq84.vGravatar Jason Gross2016-04-04
| | | | | | | | | | | | | | | | We no longer need to redefine `refine` (it now shelves by default). Also clean up `constructor` a bit.
| * | | Add compatibility Nonrecursive Elimination SchemesGravatar Jason Gross2016-04-04
| | | |
* | | | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-01-21
|\| | |
| * | | Update copyright headers.Gravatar Maxime Dénès2016-01-20
| | | |