summaryrefslogtreecommitdiff
path: root/test-suite/failure/universes-sections1.v
blob: c4eef34b1e09d1912ab9e8bdb6cfa492ef378612 (plain)
1
2
3
4
5
6
7
8
(* Check that constraints on definitions are preserved by discharging *)

Section A.
  Definition Type2 := Type.
  Definition Type1 := Type : Type2.
End A.

Definition Inconsistency := Type2 : Type1.