aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-04-15 22:21:34 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-04-15 22:21:34 +0000
commita620103f70b8805359167773a2a4fc7e2b0e38f1 (patch)
tree5c88c17b53717f4d4508383c4d3f369a63a655e8 /theories/ZArith
parente1f5180e88bf02a22c954ddbdcbdfeb168d264a6 (diff)
Fixing typo in previous commit r15180.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15181 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/Znumtheory.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Znumtheory.v b/theories/ZArith/Znumtheory.v
index 2d4bfb2e3..814b67322 100644
--- a/theories/ZArith/Znumtheory.v
+++ b/theories/ZArith/Znumtheory.v
@@ -633,7 +633,7 @@ Lemma prime_mult :
forall p:Z, prime p -> forall a b:Z, (p | a * b) -> (p | a) \/ (p | b).
Proof.
intro p; simple induction 1; intros.
- case (Zdivide_dec p a); nintuition.
+ case (Zdivide_dec p a); intuition.
right; apply Gauss with a; auto with zarith.
Qed.