教coq检查终止

Jas*_* Hu 3 termination coq totality

与许多其他人不同,Coq接受可选的显式参数,该参数可用于指示固定点定义的递减结构.

来自Gallina规范,1.3.4,

Fixpoint ident params {struct ident0 } : type0 := term0
Run Code Online (Sandbox Code Playgroud)

定义语法.但是从中我们已经知道它必须是一个标识符,而不是一般的衡量标准.

然而,一般来说,存在递归函数,终止不是很明显,或者实际上是,但终止检查器很难找到减少的结构.例如,以下程序交错两个列表,

Fixpoint interleave (A : Set) (l1 l2 : list A) : list A :=
  match l1 with
  | [] => []
  | h :: t => h :: interleave l2 t
  end
Run Code Online (Sandbox Code Playgroud)

这个功能明显终止,而Coq无法弄明白.原因既不是也l1没有l2减少每个周期.但是,如果我们考虑一个被定义为的措施length l1 + length l2呢?然后,此度量明显减少每次递归.

所以我的问题是,在复杂的情况下,代码不能直接以终止可检查的方式组织,你如何教育coq并说服它接受修复点定义?

Ant*_*nov 9

你有多个选项,最后归结为结构递归.

前言

From Coq Require Import List.
Import ListNotations.
Set Implicit Arguments.
Run Code Online (Sandbox Code Playgroud)

结构递归

有时您可以以结构递归的方式重构算法:

Fixpoint interleave1 {A} (l1 l2 : list A) {struct l1} : list A :=
  match l1, l2 with
  | [], _ => l2
  | _, [] => l1
  | h1 :: t1, h2 :: t2 => h1 :: h2 :: interleave1 t1 t2
  end.
Run Code Online (Sandbox Code Playgroud)

顺便提一下,在某些情况下,您可以使用嵌套fixes 的技巧- 请参阅Ackermann函数的这个定义(它不适用于它Fixpoint).

Program Fixpoint

您可以使用Program Fixpoint机制让您自然地编写程序,然后证明它始终终止.

From Coq Require Import Program Arith.

Program Fixpoint interleave2 {A} (l1 l2 : list A) 
  {measure (length l1 + length l2)} : list A :=
  match l1 with
  | [] => l2
  | h :: t => h :: interleave2 l2 t
  end.
Next Obligation. simpl; rewrite Nat.add_comm; trivial with arith. Qed.
Run Code Online (Sandbox Code Playgroud)

Function

另一种选择是使用Function与之相比可能有些限制的命令Program Fixpoint.您可以在此处找到有关其差异的更多信息.

From Coq Require Recdef.

Definition sum_len {A} (ls : (list A * list A)) : nat :=
  length (fst ls) + length (snd ls).

Function interleave3 {A} (ls : (list A * list A))
  {measure sum_len ls} : list A :=
  match ls with
  | ([], _) => []
  | (h :: t, l2) => h :: interleave3 (l2, t)
  end.
Proof.
  intros A ls l1 l2 h t -> ->; unfold sum_len; simpl; rewrite Nat.add_comm; trivial with arith.
Defined.
Run Code Online (Sandbox Code Playgroud)

方程式插件

这是一个外部插件,它解决了在Coq中定义函数的许多问题,包括依赖类型和终止.

From Equations Require Import Equations.

Equations interleave4 {A} (l1 l2 : list A) : list A :=
interleave4 l1 l2 by rec (length l1 + length l2) lt :=
interleave4 nil l2 := l2;
interleave4 (cons h t) l2 := cons h (interleave4 l2 t).
Next Obligation. rewrite Nat.add_comm; trivial with arith. Qed.
Run Code Online (Sandbox Code Playgroud)

如果您应用此修复程序,上面的代码.

Fix/ Fix_F_2组合者

如果您按照此问题中有关mergeSort功能的链接,您可以了解有关此(手动)方法的更多信息.顺便说一下,如果你应用我之前提到的嵌套技巧,mergeSort可以不使用函数定义函数.这是一个使用组合器的解决方案, 因为我们有两个参数,而不是像:FixfixFix_F_2mergeSort

Definition ordering {A} (l1 l2 : list A * list A) : Prop :=
  length (fst l1) + length (snd l1) < length (fst l2) + length (snd l2).

Lemma ordering_wf' {A} : forall (m : nat) (p : list A * list A),
    length (fst p) + length (snd p) <= m -> Acc (@ordering A) p.
Proof.
  unfold ordering; induction m; intros p H; constructor; intros p'.
  - apply Nat.le_0_r, Nat.eq_add_0 in H as [-> ->].
    intros contra%Nat.nlt_0_r; contradiction.
  - intros H'; eapply IHm, Nat.lt_succ_r, Nat.lt_le_trans; eauto.
Defined.

Lemma ordering_wf {A} : well_founded (@ordering A).
Proof. now red; intro ; eapply ordering_wf'. Defined.

(* it's in the stdlib but unfortunately opaque -- this blocks evaluation *)
Lemma destruct_list {A} (l : list A) :
  { x:A & {tl:list A | l = x::tl} } + { l = [] }.
Proof.
  induction l as [|h tl]; [right | left]; trivial.
  exists h, tl; reflexivity.
Defined.

Definition interleave5 {A} (xs ys : list A) : list A.
  refine (Fix_F_2 (fun _ _ => list A)
    (fun (l1 l2 : list A)
       (interleave : (forall l1' l2', ordering (l1', l2') (l1, l2) -> list A)) =>
       match destruct_list l1 with
       | inright _ => l2
       | inleft pf => let '(existT _ h (exist _ tl eq)) := pf in
                     h :: interleave l2 tl _
       end) (ordering_wf (xs,ys))).
Proof. unfold ordering; rewrite eq, Nat.add_comm; auto.
Defined.
Run Code Online (Sandbox Code Playgroud)

评估测试

Check eq_refl : interleave1 [1;2;3] [4;5;6] = [1;4;2;5;3;6].
Check eq_refl : interleave2 [1;2;3] [4;5;6] = [1;4;2;5;3;6].
Check eq_refl : interleave3 ([1;2;3], [4;5;6]) = [1;4;2;5;3;6].
Fail Check eq_refl : interleave4 [1;2;3] [4;5;6] = [1;4;2;5;3;6]. (* Equations plugin *)
Check eq_refl : interleave5 [1;2;3] [4;5;6] = [1;4;2;5;3;6].
Run Code Online (Sandbox Code Playgroud)

练习:如果你注释出destruct_list引理,最后一次检查会发生什么?