4 vector coq idris convoy-pattern
在一些依赖类型的语言(例如Idris)中实现向量添加是相当简单的.根据维基百科上的示例:
import Data.Vect
%default total
pairAdd : Num a => Vect n a -> Vect n a -> Vect n a
pairAdd Nil Nil = Nil
pairAdd (x :: xs) (y :: ys) = x + y :: pairAdd xs ys
Run Code Online (Sandbox Code Playgroud)
(注意Idris的整体检查器如何自动推断添加Nil
和非Nil
向量是逻辑上不可能的.)
我正在尝试使用自定义向量实现在Coq中实现等效功能,尽管与官方Coq库中提供的非常相似:
Set Implicit Arguments.
Inductive vector (X : Type) : nat -> Type :=
| vnul : vector X 0
| vcons {n : nat} (h : X) (v : vector X n) : vector X (S n).
Arguments vnul [X].
Fixpoint vpadd {n : nat} (v1 v2 : vector nat n) : vector nat n :=
match v1 with
| vnul => vnul
| vcons _ x1 v1' =>
match v2 with
| vnul => False_rect _ _
| vcons _ x2 v2' => vcons (x1 + x2) (vpadd v1' v2')
end
end.
Run Code Online (Sandbox Code Playgroud)
当Coq尝试检查时vpadd
,会产生以下错误:
Error:
In environment
vpadd : forall n : nat, vector nat n -> vector nat n -> vector nat n
[... other types]
n0 : nat
v1' : vector nat n0
n1 : nat
v2' : vector nat n1
The term "v2'" has type "vector nat n1" while it is expected to have type "vector nat n0".
Run Code Online (Sandbox Code Playgroud)
请注意,我False_rect
用来指定不可能的情况,否则整体检查不会通过.然而,由于某种原因,类型检查不管理统一n0
使用n1
.
我究竟做错了什么?
在普通的Coq中不可能如此轻松地实现这个功能:你需要使用护航模式重写你的功能.前一段时间有一个类似的问题.这个想法是你需要让你的match
返回函数,以传播索引之间的关系:
Set Implicit Arguments.
Inductive vector (X : Type) : nat -> Type :=
| vnul : vector X 0
| vcons {n : nat} (h : X) (v : vector X n) : vector X (S n).
Arguments vnul [X].
Definition vhd (X : Type) n (v : vector X (S n)) : X :=
match v with
| vcons _ h _ => h
end.
Definition vtl (X : Type) n (v : vector X (S n)) : vector X n :=
match v with
| vcons _ _ tl => tl
end.
Fixpoint vpadd {n : nat} (v1 v2 : vector nat n) : vector nat n :=
match v1 in vector _ n return vector nat n -> vector nat n with
| vnul => fun _ => vnul
| vcons _ x1 v1' => fun v2 => vcons (x1 + vhd v2) (vpadd v1' (vtl v2))
end v2.
Run Code Online (Sandbox Code Playgroud)
归档时间: |
|
查看次数: |
473 次 |
最近记录: |