(* Check a few naming heuristics based on types *)
(* was buggy for types names _something *)
Inductive _foo :=.
Lemma bob : (sigT (fun x : nat => _foo)) -> _foo.
destruct 1.
exact _f.
Abort.
Inductive _'Foo :=.
Lemma bob : (sigT (fun x : nat => _'Foo)) -> _'Foo.
destruct 1.
exact _'f.
Abort.
Inductive ____ :=.
Lemma bob : (sigT (fun x : nat => ____)) -> ____.
destruct 1.
exact x0.
Abort.
¤ Dauer der Verarbeitung: 0.47 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.
|