aboutsummaryrefslogtreecommitdiff
path: root/coqprime/Coqprime/ZCmisc.v
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-20 16:04:12 +0100
committerGravatar Andres Erbsen <andreser@mit.edu>2017-11-20 10:04:12 -0500
commitcaa187ddaa5e10f289c59b85844d7bc58817641b (patch)
tree4c1a4f9bb0d920ab3b74be77ed875e302bbca471 /coqprime/Coqprime/ZCmisc.v
parent3d2e80e1c91fd06197236405740e6b115b4addc4 (diff)
Remove obsolete syntax for locality. (#270)
This is preparing the landing of https://github.com/coq/coq/pull/1049. For now, I'm duplicating this patch which was already done upstream in CoqPrime, but please consider removing this ad-hoc copy (see discussion on PR #269).
Diffstat (limited to 'coqprime/Coqprime/ZCmisc.v')
-rw-r--r--coqprime/Coqprime/ZCmisc.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/coqprime/Coqprime/ZCmisc.v b/coqprime/Coqprime/ZCmisc.v
index 67709a146..ee6881849 100644
--- a/coqprime/Coqprime/ZCmisc.v
+++ b/coqprime/Coqprime/ZCmisc.v
@@ -7,7 +7,7 @@
(*************************************************************)
Require Export ZArith.
-Open Local Scope Z_scope.
+Local Open Scope Z_scope.
Coercion Zpos : positive >-> Z.
Coercion Z_of_N : N >-> Z.
@@ -88,10 +88,10 @@ Lemma Ppred_Zminus : forall p, 1< Zpos p -> (p-1)%Z = Ppred p.
Proof. destruct p;simpl;trivial. intros;elimtype False;omega. Qed.
-Open Local Scope positive_scope.
+Local Open Scope positive_scope.
Delimit Scope P_scope with P.
-Open Local Scope P_scope.
+Local Open Scope P_scope.
Definition is_lt (n m : positive) :=
match (n ?= m) with