aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zdiv.v
diff options
context:
space:
mode:
authorGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-11-01 16:46:00 +0000
committerGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-11-01 16:46:00 +0000
commit96da00b87ef2d4238fc550900e0c8f6762772810 (patch)
tree6114ef107770fd4f975f634ea05d865bdfda8b16 /theories/ZArith/Zdiv.v
parentaa0fa131bb0c5f8239644faf7a5a3069a337bb2f (diff)
Adding Qround.v (and helper lemmas and hints)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10282 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zdiv.v')
-rw-r--r--theories/ZArith/Zdiv.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index 57b0fa15c..57c0af02f 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -480,6 +480,17 @@ Proof.
ring.
Qed.
+Lemma Z_div_1 : forall z:Z, (z/1 = z)%Z.
+Proof.
+intros z.
+set (z':=z).
+unfold z' at 1.
+replace z with (0 + z*1)%Z by ring.
+rewrite (Z_div_plus 0 z 1);[reflexivity|constructor].
+Qed.
+
+Hint Resolve Z_div_1 : zarith.
+
Lemma Z_div_exact_1 : forall a b:Z, b > 0 -> a = b * (a / b) -> a mod b = 0.
intros a b Hb; generalize (Z_div_mod a b Hb); unfold Zmod, Zdiv in |- *.
case (Zdiv_eucl a b); intros q r; omega.