Set Primitive Projections.
Record foo := mkFoo { proj1 : bool; proj2 : bool }.
Definition x := mkFoo true false.
Definition proj x := proj2 x.
Lemma oops : proj = fun x => proj1 x.
Proof. Fail native_compute; reflexivity. Abort.
(*
Lemma bad : False.
assert (proj1 x = proj x).
rewrite oops; reflexivity.
discriminate.
Qed.
Print Assumptions bad.
*)
¤ Dauer der Verarbeitung: 0.17 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.
|