From caa187ddaa5e10f289c59b85844d7bc58817641b Mon Sep 17 00:00:00 2001 From: Maxime Dénès Date: Mon, 20 Nov 2017 16:04:12 +0100 Subject: 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). --- coqprime/Coqprime/ZCmisc.v | 6 +++--- 1 file changed, 3 insertions(+), 3 deletions(-) (limited to 'coqprime/Coqprime/ZCmisc.v') 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 -- cgit v1.2.3