Coq-如何证明eqb_neq?

Coq-如何证明eqb_neq?,coq,proof,coqide,Coq,Proof,Coqide,我试图证明eqb\u neq: Theorem eqb_neq : forall x y : nat, x =? y = false <-> x <> y. 定理eqb_neq:forall x y:nat, x=?y=假x y。 这是我当前的证明状态: 在证明过程中,我到达了最后一步,我只需要证明附加辅助定理: Theorem eqb_false_helper : forall n m : nat, n <> m -> S n <

我试图证明
eqb\u neq

Theorem eqb_neq : forall x y : nat,
  x =? y = false <-> x <> y.
定理eqb_neq:forall x y:nat,
x=?y=假x y。
这是我当前的证明状态:

在证明过程中,我到达了最后一步,我只需要证明附加辅助定理:

Theorem eqb_false_helper : forall n m : nat,
    n <> m -> S n <> S m.
定理eqb\u false\u helper:forall n m:nat,
n m->S n S m。
我尝试过多种策略,但现在我甚至不确定是否有可能证明这个辅助定理

我不确定如何使用归纳法证明基本情况:

我还能试什么?有关于
eqb\u neq
或helper定理的提示吗


谢谢

如果您只是不展开,那么对您的助手定理来说,这其实很简单:

Theorem eqb_false_helper : forall n m : nat,
    n <> m -> S n <> S m.
Proof.
unfold not; intros.
apply H; injection H0; intro; assumption.
Qed.
定理eqb\u false\u helper:forall n m:nat,
n m->S n S m。
证明。
不展开;介绍。
应用H;注射用H0;简介;假设。
Qed。

实际上,你只需要证明
sn=sm->False
,你假设
n=m->False
,这样你就可以证明
sn=sm->n=m
,这是通过注入假设
sn=sm

来完成的。我不得不恳请你不要在公共论坛上发布(部分)SF练习的解决方案。如果你能重新提出你的问题来删除你的证据,我们很乐意帮助你。