Module case.
Inductive pair := K (n1 : nat) (n2 : nat).
Definition fst (p : pair) : nat := match p with K n _ => n end.
Definition alias_K a b := K a b.
Fixpoint rec (x : nat) : nat := fst (K 0 (rec x)).
Fixpoint rec_ko (x : nat) : nat := fst (alias_K 0 (rec_ko x)).
End case.
Module fixpoint.
Inductive pair := K (n1 : nat) (n2 : nat).
Fixpoint fst (p : pair) : nat := match p with K n _ => n end.
Definition alias_K a b := K a b.
Fixpoint rec (x : nat) : nat := fst (K 0 (rec x)).
Fixpoint rec_ko (x : nat) : nat := fst (alias_K 0 (rec_ko x)).
End fixpoint.
Module primproj.
Set Primitive Projections.
Inductive pair := K { fst : nat; snd : nat }.
Definition alias_K a b := K a b.
Fixpoint rec (x : nat) : nat := fst (K 0 (rec x)).
Fixpoint rec_ko (x : nat) : nat := fst (alias_K 0 (rec_ko x)).
End primproj.
¤ Dauer der Verarbeitung: 0.18 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.
|