我正在编写一种玩具语言,其中AST中的节点可以包含任意数量的子节点(Num
有0,Arrow
有2等)。你可以称这些运营商。另外,AST中的一个节点可能是“聚焦”的。如果数据类型具有焦点,我们会将数据类型编入索引Z
,如果数据类型没有,则为H
。
我需要有关代码的一些部分的建议。希望一下子就可以问所有这些,因为它们是相关的。
您如何定义一个焦点InternalZ
的内部节点类型?现在我说“我们有S n
个孩子 - n
他们没有聚焦,一个(在某个给定的索引处)聚焦。一个稍微更直观的选项(看起来像拉链)将是{ {1}}。我知道我不想处理这种添加。
精炼类型:在InternalZ : forall n m, arityCode (n + 1 + m) -> Vector.t (t H) n -> t Z -> Vector.t (t H) m -> t Z
中的两个有趣案例中,我比较了两个eq
s(子项数)。如果它们是相同的,我应该能够“强制”n
和arityCode
s具有相同的类型。现在我用两个引理来攻击这个。我该怎么做呢?似乎Adam Chlipala的"convoy pattern"可能有所帮助,但我无法弄清楚如何。
如果我取消注释Vector.t
个调用之一,Coq会抱怨“无法猜测减少修正的参数。”。我理解错误,但我不确定如何规避错误。我想到的第一件事就是我可能必须根据孩子的深度来指出Vector.eqb
。
我的代码:
t
答案 0 :(得分:6)
让我们从你的第三个问题开始吧。 Vector.eqb
对其第一个参数执行嵌套递归调用。为了说服Coq这些正在减少,我们需要通过将coerceVec
替换为Qed
来使Defined
的定义透明:
Require Coq.Arith.EqNat.
Require Coq.Structures.Equalities.
Require Coq.Arith.Peano_dec.
Require Fin.
Require Vector.
Set Implicit Arguments.
Module Typ.
Import Coq.Arith.EqNat.
Import Coq.Structures.Equalities.
Import Coq.Arith.Peano_dec.
Import Fin.
Import Vector.
(* h: unfocused, z: focused *)
Inductive hz : Set := H | Z.
Inductive arityCode : nat -> Type :=
| Num : arityCode 0
| Hole : arityCode 0
| Arrow : arityCode 2
| Sum : arityCode 2
.
Definition codeEq (n : nat) (l r : arityCode n) : bool :=
match l, r with
| Num, Num => true
| Hole, Hole => true
| Arrow, Arrow => true
| Sum, Sum => true
| _, _ => false
end.
Inductive t : hz -> Type :=
| Leaf : arityCode 0 -> t H
| Cursor : t H -> t Z
| InternalH : forall n, arityCode n -> Vector.t (t H) n -> t H
| InternalZ : forall n, arityCode (S n) -> Vector.t (t H) n -> Fin.t n * t Z -> t Z
.
Lemma coerceArity (n1 n2 : nat) (pf : n1 = n2) (c1 : arityCode n1) : arityCode n2.
exact (eq_rect n1 arityCode c1 n2 pf).
Defined.
Lemma coerceVec {A : Type} {n1 n2 : nat} (pf : n1 = n2) (c1 : Vector.t A n1) : Vector.t A n2.
exact (eq_rect n1 (Vector.t A) c1 n2 pf).
Defined.
Fixpoint eq {h_or_z : hz} (ty1 ty2 : t h_or_z) : bool :=
match ty1, ty2 with
| Leaf c1, Leaf c2 => codeEq c1 c2
| Cursor ty1, Cursor ty2 => eq ty1 ty2
| @InternalH n1 c1 ty1, @InternalH n2 c2 ty2 =>
match eq_nat_dec n1 n2 with
| right _neqPrf => false
| left eqPrf =>
let c1' := coerceArity eqPrf c1 in
let ty1' := coerceVec eqPrf ty1 in
codeEq c1' c2 && Vector.eqb _ eq ty1' ty2
end
| @InternalZ n1 c1 v1 (l1, f1), @InternalZ n2 c2 v2 (l2, f2) =>
match eq_nat_dec n1 n2 with
| right _neqPrf => false
| left eqPrf =>
let eqPrf' := f_equal S eqPrf in
let c1' := coerceArity eqPrf' c1 in
let v1' := coerceVec eqPrf v1 in
codeEq c1' c2 && Vector.eqb _ eq v1' v2 && Fin.eqb l1 l2 && eq f1 f2
end
| _, _ => false
end.
End Typ.
至于你的第二个问题:一般来说,你确实需要使用相等证明来实现强制转换操作,就像使用coerceVec
一样。但是,在这种特殊情况下,更容易避免使用具有不同索引的元素的强制转换和写入比较函数:
Require Coq.Arith.EqNat.
Require Coq.Structures.Equalities.
Require Coq.Arith.Peano_dec.
Require Fin.
Require Vector.
Set Implicit Arguments.
Module Typ.
Import Coq.Arith.EqNat.
Import Coq.Structures.Equalities.
Import Coq.Arith.Peano_dec.
Import Fin.
Import Vector.
(* h: unfocused, z: focused *)
Inductive hz : Set := H | Z.
Inductive arityCode : nat -> Type :=
| Num : arityCode 0
| Hole : arityCode 0
| Arrow : arityCode 2
| Sum : arityCode 2
.
Definition codeEq (n1 n2 : nat) (l : arityCode n1) (r : arityCode n2) : bool :=
match l, r with
| Num, Num => true
| Hole, Hole => true
| Arrow, Arrow => true
| Sum, Sum => true
| _, _ => false
end.
Inductive t : hz -> Type :=
| Leaf : arityCode 0 -> t H
| Cursor : t H -> t Z
| InternalH : forall n, arityCode n -> Vector.t (t H) n -> t H
| InternalZ : forall n, arityCode (S n) -> Vector.t (t H) n -> Fin.t n * t Z -> t Z
.
Fixpoint eq {h_or_z : hz} (ty1 ty2 : t h_or_z) : bool :=
match ty1, ty2 with
| Leaf c1, Leaf c2 => codeEq c1 c2
| Cursor ty1, Cursor ty2 => eq ty1 ty2
| @InternalH n1 c1 ty1, @InternalH n2 c2 ty2 =>
match eq_nat_dec n1 n2 with
| right _neqPrf => false
| left eqPrf =>
codeEq c1 c2 && Vector.eqb _ eq ty1 ty2
end
| @InternalZ n1 c1 v1 (l1, f1), @InternalZ n2 c2 v2 (l2, f2) =>
match eq_nat_dec n1 n2 with
| right _neqPrf => false
| left eqPrf =>
codeEq c1 c2 && Vector.eqb _ eq v1 v2 && Fin.eqb l1 l2 && eq f1 f2
end
| _, _ => false
end.
End Typ.
最难和最开放的问题是第一个问题。我认为对类型进行建模的最简单方法是将其拆分为两种:一种原始语法树,以及一种由树索引的路径。例如:
Require Fin.
Require Vector.
Set Implicit Arguments.
Module Typ.
Inductive arityCode : nat -> Type :=
| Num : arityCode 0
| Hole : arityCode 0
| Arrow : arityCode 2
| Sum : arityCode 2
.
Inductive t : Type :=
| Node : forall n, arityCode n -> Vector.t t n -> t.
Inductive path : t -> Type :=
| Here : forall n (c : arityCode n) (v : Vector.t t n), path (Node c v)
| There : forall n (c : arityCode n) (v : Vector.t t n) (i : Fin.t n),
path (Vector.nth v i) -> path (Node c v).
End Typ.
此处,path tree
表示树tree
中的索引类型。
Coq社区经常就如何以及何时使用依赖类型存在分歧。在这种特殊情况下,我认为将一个t
类型的原始语法树和一个非依赖类型path
的路径放入树中会更容易。您可以定义表示相对于树的路径的良构性的谓词,并在您关注的函数遵循良构的概念之后证明。在这种情况下我发现这更灵活,因为你不必担心在你的函数中操纵类型索引并推理它们(理解这意味着什么,试着说明原始Typ.eq
函数的正确性定理)。