Inductive array : Type -> Type :=
| carray : forall A, array A.
Inductive Mtac : Type -> Prop :=
| bind : forall {A B}, Mtac A -> (A -> Mtac B) -> Mtac B
| array_make : forall {A}, A -> Mtac (array A).
Definition Ref := array.
Definition ref : forall {A}, A -> Mtac (Ref A) :=
fun A x=> array_make x.
Check array Type.
Check fun A : Type => Ref A.
Definition abs_val (a : Type) :=
bind (ref a) (fun r : array Type => array_make tt).
¤ Dauer der Verarbeitung: 0.26 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.
|