aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
Diffstat (limited to 'theories')
-rw-r--r--theories/ZArith/Zcomplements.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/theories/ZArith/Zcomplements.v b/theories/ZArith/Zcomplements.v
index 5b3e16968..d5075ffb6 100644
--- a/theories/ZArith/Zcomplements.v
+++ b/theories/ZArith/Zcomplements.v
@@ -18,6 +18,8 @@ Open Local Scope Z_scope.
(**********************************************************************)
(* Properties of comparison on Z *)
+Set Implicit Arguments.
+
Theorem Zcompare_Zmult_right : (x,y,z:Z)` z>0` -> `x ?= y`=`x*z ?= y*z`.
Intros; Apply Zcompare_egal_dec;
@@ -139,10 +141,10 @@ Elim (H `|m|`);Intros;Auto with zarith.
Elim (Zabs_dec m);Intro eq;Rewrite eq;Trivial.
Qed.
-(** To do case analysis over the sign of [z] *)
-
Unset Implicit Arguments.
+(** To do case analysis over the sign of [z] *)
+
Lemma Zcase_sign : (x:Z)(P:Prop)
(`x=0` -> P) ->
(`x>0` -> P) ->