aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/omega
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:26:26 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:26:26 +0000
commitaca0bb7546310d87146d27f16b1e98699a23e085 (patch)
tree4eb12f65e66e6acf9361e72488a59ea141c762c7 /contrib/omega
parentce0730a894791ea19a2ac372a63c94a141102cf8 (diff)
Restructuration ZArith
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4879 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/omega')
-rw-r--r--contrib/omega/OmegaLemmas.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/contrib/omega/OmegaLemmas.v b/contrib/omega/OmegaLemmas.v
index 98922f3fd..c29224069 100644
--- a/contrib/omega/OmegaLemmas.v
+++ b/contrib/omega/OmegaLemmas.v
@@ -78,7 +78,7 @@ Lemma OMEGA8:
Intros x y H1 H2 H3; Elim (Zle_lt_or_eq ZERO x H1); [
Intros H4; Absurd (Zlt ZERO x); [
- Change (Zge ZERO x); Apply Zle_ge; Apply (Zsimpl_le_plus_l y);
+ Change (Zge ZERO x); Apply Zle_ge; Apply Zsimpl_le_plus_l with y;
Rewrite -> H3; Rewrite Zplus_inverse_r; Rewrite Zero_right; Assumption
| Assumption]
| Intros H4; Rewrite -> H4; Trivial with arith].