aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/auxiliary.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-05 10:58:08 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-05 10:58:08 +0000
commit4dbf6842e0b2b43c5f8c15817942dfecaab5cd2e (patch)
treef81b47df039aed8471726bfb635b6a675602ecab /theories/ZArith/auxiliary.v
parent21cd39996cabdf280f4cc99557c54f6c7c73bbc8 (diff)
petits changements afin de profiter du nouveau Rewrite/in
(l'unification marche mieux) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2512 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/auxiliary.v')
-rw-r--r--theories/ZArith/auxiliary.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/auxiliary.v b/theories/ZArith/auxiliary.v
index e6edf81a5..b6505d6bb 100644
--- a/theories/ZArith/auxiliary.v
+++ b/theories/ZArith/auxiliary.v
@@ -713,7 +713,7 @@ Theorem OMEGA20:
(x,y,z:Z)(Zne x ZERO) -> (y=ZERO) -> (Zne (Zplus x (Zmult y z)) ZERO).
Unfold Zne not; Intros x y z H1 H2 H3; Apply H1; Rewrite H2 in H3;
-Simpl in H3; Rewrite (Zero_right x) in H3; Trivial with arith.
+Simpl in H3; Rewrite Zero_right in H3; Trivial with arith.
Save.
Definition fast_Zplus_sym :=