aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-10 09:25:54 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-10 09:25:54 +0000
commit8cc29f42843d432b949d3760b15de6bd6ab567e4 (patch)
treed3b2d0e565de2f6f41b24152d57eceb968ecc4df /theories
parent8ddd34d0fc3433c9b826ce30a2715d58b740cc72 (diff)
Finalement, encore un Simpl inutile
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@676 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-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 f1d156a70..de7ed41d3 100644
--- a/theories/Zarith/auxiliary.v
+++ b/theories/Zarith/auxiliary.v
@@ -388,7 +388,7 @@ Save.
Lemma add_x_x : (x:positive) (add x x) = (xO x).
Intros p; Apply convert_intro; Simpl; Rewrite convert_add;
-Simpl; Rewrite ZL6; Trivial with arith.
+Rewrite ZL6; Trivial with arith.
Save.
Theorem Zcompare_Zmult_compatible :