From a46ccd71539257bb55dcddd9ae8510856a5c9a16 Mon Sep 17 00:00:00 2001 From: letouzey Date: Thu, 5 Jul 2012 16:56:28 +0000 Subject: Open Local Scope ---> Local Open Scope, same with Notation and alii git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15517 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Bool/Bool.v | 2 +- theories/Bool/Bvector.v | 2 +- theories/Bool/Zerob.v | 2 +- 3 files changed, 3 insertions(+), 3 deletions(-) (limited to 'theories/Bool') diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v index 92a584256..79a719a1f 100644 --- a/theories/Bool/Bool.v +++ b/theories/Bool/Bool.v @@ -754,7 +754,7 @@ Notation "a &&& b" := (if a then b else false) Notation "a ||| b" := (if a then true else b) (at level 50, left associativity) : lazy_bool_scope. -Open Local Scope lazy_bool_scope. +Local Open Scope lazy_bool_scope. Lemma andb_lazy_alt : forall a b : bool, a && b = a &&& b. Proof. diff --git a/theories/Bool/Bvector.v b/theories/Bool/Bvector.v index 0c2181638..2f904c81b 100644 --- a/theories/Bool/Bvector.v +++ b/theories/Bool/Bvector.v @@ -13,7 +13,7 @@ Require Vector. Export Vector.VectorNotations. Require Import Minus. -Open Local Scope nat_scope. +Local Open Scope nat_scope. (** We build bit vectors in the spirit of List.v. diff --git a/theories/Bool/Zerob.v b/theories/Bool/Zerob.v index bac4c0d69..5689bf50d 100644 --- a/theories/Bool/Zerob.v +++ b/theories/Bool/Zerob.v @@ -9,7 +9,7 @@ Require Import Arith. Require Import Bool. -Open Local Scope nat_scope. +Local Open Scope nat_scope. Definition zerob (n:nat) : bool := match n with -- cgit v1.2.3