aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_093.v
Commit message (Collapse)AuthorAge
* 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.
* Univs: minor fixes to test-suite filesGravatar Matthieu Sozeau2015-10-02
| | | | 108 used an implicit lowering to Prop.
* Explicit universes allow to write liftings explicitely. Implicit lifting ↵Gravatar Matthieu Sozeau2014-06-17
would change the theory non-trivially.