diff options
author | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-12-15 19:48:24 +0000 |
---|---|---|
committer | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-12-15 19:48:24 +0000 |
commit | 3675bac6c38e0a26516e434be08bc100865b339b (patch) | |
tree | 87f8eb1905c7b508dea60b1e216f79120e9e772d /contrib/omega/OmegaLemmas.v | |
parent | c881bc37b91a201f7555ee021ccb74adb360d131 (diff) |
modif existentielle (exists | --> exists ,) + bug d'affichage des pt fixes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5099 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/omega/OmegaLemmas.v')
-rw-r--r-- | contrib/omega/OmegaLemmas.v | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/contrib/omega/OmegaLemmas.v b/contrib/omega/OmegaLemmas.v index 61747028e..1c7428605 100644 --- a/contrib/omega/OmegaLemmas.v +++ b/contrib/omega/OmegaLemmas.v @@ -12,7 +12,7 @@ Require Import ZArith_base. (** These are specific variants of theorems dedicated for the Omega tactic *) -Lemma new_var : forall x:Z, exists y : Z | x = y. +Lemma new_var : forall x:Z, exists y : Z, x = y. intros x; exists x; trivial with arith. Qed. @@ -266,4 +266,4 @@ Definition fast_Zred_factor5 (x y:Z) (P:Z -> Prop) (H:P y) := eq_ind_r P H (Zred_factor5 x y). Definition fast_Zred_factor6 (x:Z) (P:Z -> Prop) (H:P (x + 0)%Z) := - eq_ind_r P H (Zred_factor6 x).
\ No newline at end of file + eq_ind_r P H (Zred_factor6 x). |