aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Znumtheory.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-24 20:48:15 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-24 20:48:15 +0000
commit72add906154ce22894a41cf04543a7c096456e09 (patch)
tree5dd21c4198789c6791b845008120c71b2058c95e /theories/ZArith/Znumtheory.v
parent2337b9bfc662981a2630df8c173d54b32fa2b2b6 (diff)
Tauto breaking not only binary "conjunctions" seems like a bad idea
after all... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11259 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Znumtheory.v')
-rw-r--r--theories/ZArith/Znumtheory.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/theories/ZArith/Znumtheory.v b/theories/ZArith/Znumtheory.v
index f4e5bfc15..93ec1081b 100644
--- a/theories/ZArith/Znumtheory.v
+++ b/theories/ZArith/Znumtheory.v
@@ -521,8 +521,7 @@ Qed.
Lemma Zis_gcd_mult :
forall a b c d:Z, Zis_gcd a b d -> Zis_gcd (c * a) (c * b) (c * d).
Proof.
- intros a b c d; simple induction 1; constructor.
- intuition. intuition. intros.
+ intros a b c d; simple induction 1; constructor; intuition.
elim (Zis_gcd_bezout a b d H). intros.
elim H3; intros.
elim H4; intros.