证明不到

时间:2013-03-17 17:00:02

标签: logic coq

我试图在Coq中证明关于less_than的一些定理。我 使用这个归纳定义:

Inductive less_than : nat->nat->Prop :=
   | lt1 : forall a, less_than O (S a)
   | lt2 : forall a b, less_than a b -> less_than a (S b)
   | lt3 : forall a b, less_than a b -> less_than (S a) (S b).

我总是需要显示lt3的反转,

Lemma inv_lt3, forall a b, less_than (S a) (S b) -> less_than a b.
Proof.
   ???

我被困住了,如果有人提示如何继续,我将非常感激。

(我对less_than的归纳定义是否有问题?)

谢谢!

1 个答案:

答案 0 :(得分:5)

首先,你对less_than的定义有点不幸,因为第二个构造函数是多余的。您应该考虑切换到更简单的方法:

Inductive less_than : nat -> nat -> Prop :=
| ltO : forall a, less_than O (S a)
| ltS : forall a b, less_than a b -> less_than (S a) (S b)
.

然后反演将匹配coq的反演,使你的证明变得微不足道:

Lemma inv_ltS: forall a b, less_than (S a) (S b) -> less_than a b.
Proof. now inversion 1. Qed.

第二个条款是多余的,因为对于每一对(a, b) st。如果您需要less_than a b的证明,则可以始终应用lt3 a次,然后应用lt1。你的lt2实际上是另外两个构造函数的结果:

Ltac inv H := inversion H; subst; clear H; try tauto.

(* there is probably an easier way to do that? *)
Lemma lt2 : forall a b, less_than a b -> less_than a (S b).
Proof.
  intros a b. revert a. induction b; intros.
  inv H.
  inv H.
  apply ltO.
  apply ltS. now apply IHb.
Qed.

现在,如果您真的希望保留您的特定定义,请按照以下方式尝试证明:

Lemma inv_lt: forall a b, less_than (S a) (S b) -> less_than a b.
Proof.
  induction b; intros.
  inv H. inv H2.
  inv H. apply lt2. now apply IHb.
Qed.