aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-05 13:43:43 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-05 13:43:43 +0000
commitafda8af89cd10a31419da859ff136fd1c4c0fa22 (patch)
treea7774fe054c7f556204d35a2f7113dc9b96195da /theories/ZArith
parentcefe8d9e1acc211a505808703dda93acac050ced (diff)
Zabs_Zsgn
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4307 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/zarith_aux.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/ZArith/zarith_aux.v b/theories/ZArith/zarith_aux.v
index 936468fef..81c87f7c1 100644
--- a/theories/ZArith/zarith_aux.v
+++ b/theories/ZArith/zarith_aux.v
@@ -77,9 +77,9 @@ Proof.
Destruct x;Intros;Rewrite Zmult_sym;Auto with arith.
Qed.
-Lemma Zabs_Zsgn: (x:Z)(Zabs x)=(Zmult (Zsgn x) x).
+Lemma Zabs_Zsgn: (x:Z)(Zmult (Zabs x) (Zsgn x))=x.
Proof.
-Destruct x;Intros;Auto with arith.
+Destruct x;Intros; Rewrite Zmult_sym; Auto with arith.
Qed.
(** From [nat] to [Z] *)