Set Primitive Projections.
CoInductive stream A := { hd : A; tl : stream A }.
CoFixpoint ticks (n : nat) : stream unit := {| hd := tt; tl := ticks n |}.
Lemma expand : exists n : nat, (ticks n) = (ticks n).(tl _).
Proof.
eexists.
(* Set Debug Tactic Unification. *)
(* Set Debug RAKAM. *)
reflexivity.
Abort.
¤ Dauer der Verarbeitung: 0.16 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.
|