blob: 7d1d3ee692b56c826bfe4abbf0a79e0b7df14561 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
|
(* Check that arguments of impredicative types are not considered
subterms for the guard condition (an example by Thierry Coquand) *)
Inductive I : Prop :=
| C: (forall P:Prop, P->P) -> I.
Definition i0 := C (fun _ x => x).
Fail Definition Paradox : False :=
(fix ni i : False :=
match i with
| C f => ni (f _ i)
end) i0.
|