(* Not considering singleton template-polymorphic inductive types as
propositions for injection/inversion *)
(* This is also #4560 and #6273 *)
Inductive foo := foo_1.
Goal forall (a b : foo), Some a = Some b -> a = b.
Proof.
intros a b H.
inversion H.
reflexivity.
Qed.
(* Check that Prop is not concerned *)
Inductive bar : Prop := bar_1.
Goal
forall (a b : bar),
Some a = Some b ->
a = b.
Proof.
intros a b H.
inversion H.
Fail reflexivity.
Abort.
¤ Dauer der Verarbeitung: 0.13 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.
|