aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zdiv.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-08 14:33:00 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-08 14:33:00 +0000
commitd1be0ed0d067dc37afcc5db5e58cee5c2a89d646 (patch)
treeeb79e99e77c01d820b84fc9d4eef1e090b17cae0 /theories/ZArith/Zdiv.v
parentfee7eda39631ef33c6c3df31b3361ac53d6e945b (diff)
one forgotten compatibility lemma
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10526 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zdiv.v')
-rw-r--r--theories/ZArith/Zdiv.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index 85d2b06f6..de3b76e95 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -1033,6 +1033,11 @@ Proof.
intros; apply Z_div_same_full; auto with zarith.
Qed.
+Lemma Z_div_plus : forall a b c:Z, c > 0 -> (a + b * c) / c = a / c + b.
+Proof.
+ intros; apply Z_div_plus_full; auto with zarith.
+Qed.
+
Lemma Z_div_mult : forall a b:Z, b > 0 -> (a*b)/b = a.
Proof.
intros; apply Z_div_mult_full; auto with zarith.