aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar roconnor-blockstream <roconnor@blockstream.com>2017-06-29 17:57:05 -0400
committerGravatar GitHub <noreply@github.com>2017-06-29 17:57:05 -0400
commit79f2e62eb22318c9a2b0c96a19ef3fadd1ca781d (patch)
treeb05a666df5c87df9f3336d67aa3f9602cf99e3a3 /theories
parentf4f609f598fb4804acf272209782b60d4647cad4 (diff)
Use forall for consistency
Diffstat (limited to 'theories')
-rw-r--r--theories/ZArith/Zdiv.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index 509384104..140d1b3c8 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -508,7 +508,7 @@ Qed.
(** Unfortunately, the previous result isn't always true on negative numbers.
For instance: 3/(-2)/(-2) = 1 <> 0 = 3 / (-2*-2) *)
-Lemma Zmod_div (a b : Z) : a mod b / b = 0.
+Lemma Zmod_div : forall a b, a mod b / b = 0.
Proof.
zero_or_not b.
auto using Z.mod_div.