在一些依赖类型语言(例如 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
(请注意 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.
当 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".
请注意,我使用False_rect
指定不可能的情况,否则整体检查不会通过。但是,由于某种原因,类型检查器无法n0
与n1
.
我究竟做错了什么?