diff options
author | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-07-23 06:27:58 +0000 |
---|---|---|
committer | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-07-23 06:27:58 +0000 |
commit | 25927c9afb1c5fa62ee4af1427c85a23623fe0ae (patch) | |
tree | 58d41706f80ecd666909d30d8b8573661c52a346 /theories | |
parent | ee07024b3b3265c2764e2d6b26036a69c280cb70 (diff) |
Oops... forgot some debug code.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11247 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r-- | theories/ZArith/Znumtheory.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Znumtheory.v b/theories/ZArith/Znumtheory.v index 599d6791a..f4e5bfc15 100644 --- a/theories/ZArith/Znumtheory.v +++ b/theories/ZArith/Znumtheory.v @@ -522,7 +522,7 @@ 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. intuition. + intuition. intuition. intros. elim (Zis_gcd_bezout a b d H). intros. elim H3; intros. elim H4; intros. |