aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3559.v
Commit message (Collapse)AuthorAge
* Fix (partial) #4878: option to stop autodeclaring axiom as instance.Gravatar Gaƫtan Gilbert2017-11-28
|
* 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.
* Fixing line break in test for #3559.Gravatar Hugo Herbelin2014-09-15
|
* Fix test-suite files, and move some opened to closed.Gravatar Matthieu Sozeau2014-09-11
|
* Fix bug #3559, ensuring a canonical order of universe level quantifications whenGravatar Matthieu Sozeau2014-09-04
introducing constants (e.g. Top.1 is always before Top.2), compatible with the one used before introduction of hMaps in LMap/LSet.