Set Universe Polymorphism.
Module Type T.
Axiom foo@{u v|u < v} : Type@{v}.
End T.
Module M : T with Definition foo@{u v} := Type@{u} : Type@{v}.
Definition foo@{u v} := Type@{u} : Type@{v}.
End M.
Fail Module M' : T with Definition foo := Type.
(* Without the binder expression we have to do trickery to get the
universes in the right order. *)
Module M' : T with Definition foo := let t := Type in t.
Definition foo := let t := Type in t.
End M'.
¤ Dauer der Verarbeitung: 0.0 Sekunden
(vorverarbeitet)
¤
|
Haftungshinweis
Die Informationen auf dieser Webseite wurden
nach bestem Wissen sorgfältig zusammengestellt. Es wird jedoch weder Vollständigkeit, noch Richtigkeit,
noch Qualität der bereit gestellten Informationen zugesichert.
Bemerkung:
Die farbliche Syntaxdarstellung ist noch experimentell.
|