Require Import Coq.Program.Tactics.
(* these should not result in anomalies *)
Fail Program Lemma foo:
forall P, forall H, forall (n:nat), P n.
Fail Program Lemma foo:
forall a (P : list a -> Prop), forall H, forall (n:list a), P n.
Fail Program Lemma foo:
forall (a : Type) (P : list a -> Prop), forall H, forall (n:list a), P n.
¤ Dauer der Verarbeitung: 0.1 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.
|