3
Require Import Streams.

CoFixpoint map {X Y : Type} (f : X -> Y) (s : Stream X) : Stream Y :=
  Cons (f (hd s)) (map f (tl s)).

CoFixpoint interleave {X : Type} (s : Stream X * Stream X) : Stream X := Cons (hd (fst s)) (Cons (hd (snd s)) (interleave (tl (fst s), tl (snd s)))).

Lemma map_interleave : forall {X Y : Type} (f : X -> Y) (s1 s2 : Stream X), map f (interleave (s1, s2)) = interleave (map f s1, map f s2).
Proof.
  Fail cofix. (* error *)
Abort.

输出:

Ltac call to "cofix" failed.
Error: All methods must construct elements in coinductive types.

我不确定这意味着什么 - 两者map都是interleave直接的核心递归函数,用于构建共归纳类型的值。有什么问题?

4

1 回答 1

2

问题源于=符号代表的事实eq,它是一种归纳类型,而不是一种共归纳类型。

相反,您可以证明流map f (interleave (s1, s2))interleave (map f s1, map f s2)扩展相等。这是 Coq 参考手册的摘录(第 1.3.3 节

为了证明两个流的外延相等,s1我们s2必须构造一个无限的相等证明,即类型的无限对象EqSt s1 s2

改成后eq我们EqSt可以证明引理:

Lemma map_interleave : forall {X Y : Type} (f : X -> Y) (s1 s2 : Stream X),
  EqSt (map f (interleave (s1, s2))) (interleave (map f s1, map f s2)).
Proof.
  cofix.
  intros X Y f s1 s2.
  do 2 (apply eqst; [reflexivity |]).
  case s1 as [h1 s1], s2 as [h2 s2].
  change (tl (tl (map f (interleave (Cons h1 s1, Cons h2 s2))))) with
         (map f (interleave (s1, s2))).
  change (tl (tl (interleave (map f (Cons h1 s1), map f (Cons h2 s2))))) with
         (interleave (map f s1, map f s2)).
  apply map_interleave.
Qed.

顺便说一句,在这个CPDT 章节中可以找到许多处理协约数据类型的技巧。

于 2017-06-18T10:40:56.833 回答