blob: ec9cf44d4f20a582c2e3b18e863bf26c0a45b5a6 (
plain)
1
2
3
4
5
6
7
8
9
|
Universes i j k l.
Definition foo : Type@{j} := Type@{i}.
Definition baz : Type@{k} := Type@{l}.
Print Universes Subgraph(i j).
(* should print [i < j], not [l < k] (and not prelude universes) *)
|