(* 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.
¤ Dauer der Verarbeitung: 0.2 Sekunden
(vorverarbeitet)
¤
|
Haftungshinweis
Die Informationen auf dieser Webseite wurden
nach bestem Wissen sorgfältig zusammengestellt. Es wird jedoch weder Vollständigkeit, noch Richtigkeit,
noch Qualität der bereit gestellten Informationen zugesichert.
Bemerkung:
Die farbliche Syntaxdarstellung ist noch experimentell.
|