summaryrefslogtreecommitdiff
path: root/test-suite/failure/universes-sections2.v
blob: 34b2a11ded0fab3608a26f43280cc50712022c7d (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.

Fail Definition Inconsistency : Type1' := Type2.