From 79f2e62eb22318c9a2b0c96a19ef3fadd1ca781d Mon Sep 17 00:00:00 2001 From: roconnor-blockstream Date: Thu, 29 Jun 2017 17:57:05 -0400 Subject: Use forall for consistency --- theories/ZArith/Zdiv.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories') 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. -- cgit v1.2.3