如何证明x+;y-z=x+;(y-z)在Coq中

如何证明x+;y-z=x+;(y-z)在Coq中,coq,proof,Coq,Proof,我想证明这一点: 1 subgoals x : nat y : nat z : nat ______________________________________(1/1) x + y - z = x + (y - z) 它看起来很琐碎,但它让我很困惑,我需要它作为另一个证据 谢谢。如果你想证明的不成立,你想证明的不成立,如果你想证明的不成立,你能把问题标记为已回答吗?(单击问题旁边的复选标记)是否将问题标记为已回答?(单击问题旁边的复选标记) Require Import Omega. T

我想证明这一点:

1 subgoals
x : nat
y : nat
z : nat
______________________________________(1/1)
x + y - z = x + (y - z)
它看起来很琐碎,但它让我很困惑,我需要它作为另一个证据


谢谢。

如果你想证明的不成立,你想证明的不成立,如果你想证明的不成立,你能把问题标记为已回答吗?(单击问题旁边的复选标记)是否将问题标记为已回答?(单击问题旁边的复选标记)
Require Import Omega.
Theorem foo:
    forall x y z:nat, (x = 0 \/ z <= y) <->  x + y - z = x + (y - z).
    intros; omega.
Qed.
Require Import ZArith.
Open Scope Z.
Theorem fooZ:
    forall x y z:Z, x + y - z = x + (y - z).
    intros; omega.
Qed.