aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4121.v
Commit message (Collapse)AuthorAge
* Merge branch 'v8.6'Gravatar Pierre-Marie Pédrot2017-05-17
|\
| * remove unneeded -emacs flag to coq-prog-argsGravatar Paul Steckler2017-05-01
| |
* | Moving the Ltac plugin to a pack-based one.Gravatar Pierre-Marie Pédrot2017-02-17
|/ | | | | | | This is cumbersome, because now code may fail at link time if it's not referring to the correct module name. Therefore, one has to add corresponding open statements a the top of every file depending on a Ltac module. This includes seemingly unrelated files that use EXTEND statements.
* 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.
* Fix declarations of instances to perform restriction of universeGravatar Matthieu Sozeau2015-04-09
instances as definitions and lemmas do (fixes bug# 4121).