blob: 3f8e4446232affc6a49f549942a4a52f73d87c51 (
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 : Type2 := Type.
End A.
Fail Definition Inconsistency : Type1 := Type2.
|