summaryrefslogtreecommitdiff
path: root/test-suite/failure/universes-sections2.v
blob: 98fdbc0d1d4e3a1f200bcbb7bd1f3aeaf0187730 (plain)
1
2
3
4
5
6
7
8
9
10
(* Check that constraints on locals are preserved by discharging *)

Definition Type2 := Type.

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

Definition Inconsistency : Type1' := Type2.