diff options
Diffstat (limited to 'contrib/correctness/ProgInt.v')
| -rw-r--r-- | contrib/correctness/ProgInt.v | 6 |
1 files changed, 3 insertions, 3 deletions
diff --git a/contrib/correctness/ProgInt.v b/contrib/correctness/ProgInt.v index ec46e2de62..470162ca34 100644 --- a/contrib/correctness/ProgInt.v +++ b/contrib/correctness/ProgInt.v @@ -13,7 +13,7 @@ Require Export ZArith. Require Export ZArith_dec. -Theorem Znotzero : (x:Z){`x<>0`}+{`x=0`}. +Theorem Znotzero : forall x:Z, {x <> 0%Z} + {x = 0%Z}. Proof. -Intro x. Elim (Z_eq_dec x `0`) ; Auto. -Save. +intro x. elim (Z_eq_dec x 0); auto. +Qed.
\ No newline at end of file |
