blob: f32e0969c8176507b065d6018460a2337abd8988 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
|
(* Check let-ins in fix and Fixpoint *)
Definition foo := fix f (m : nat) (o := true) (n : nat) {struct n} :=
match n with 0 => 0 | S n' => f 0 n' end.
Fixpoint f (m : nat) (o := true) (n : nat) {struct n} :=
match n with 0 => 0 | S n' => f 0 n' end.
Definition foo' := fix f {m : nat} (o := true) (n : nat) {struct n} :=
match n with 0 => 0 | S n' => f (m:=0) n' end.
Check foo' (m:=0) 0.
Fixpoint f' {m : nat} (o := true) (n : nat) {struct n} :=
match n with 0 => 0 | S n' => f' (m:=0) n' end.
Check f' (m:=0) 0.
CoInductive Stream := { hd : nat; tl : Stream }.
Definition cofoo := cofix f (o := true) {m} := {| hd := 0; tl := f (m:=0) |}.
Check cofoo (m:=0).
CoFixpoint cof (o := true) {m} := {| hd := 0; tl := cof (m:=0) |}.
Check cof (m:=0).
Definition cofoo' := cofix f {m} (o := true) := {| hd := 0; tl := f (m:=0) |}.
Check cofoo' (m:=0).
CoFixpoint cof' {m} (o := true) := {| hd := 0; tl := cof' (m:=0) |}.
Check cof' (m:=0).
|