aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-26 11:33:55 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-26 11:33:55 +0000
commitf87c74e95b89d61cc739bde85b95b3e5055d9b96 (patch)
treef7b9246c54e977f026940ea2ca3d34a5d1628ad1
parent999d557f9733cca6b2249750622ca599ac6985c6 (diff)
'Open Local Scope' en attendant que le core_scope sache se mettre devant implicitement
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4485 85f007b7-540e-0410-9357-904b9bb8a0f7
-rwxr-xr-xtheories/Bool/Bool.v2
-rw-r--r--theories/ZArith/fast_integer.v2
2 files changed, 2 insertions, 2 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 8da809d50..0e254c8e5 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -178,7 +178,7 @@ Infix "&&" andb (at level 3, no associativity) : bool_scope
Notation "- b" := (negb b) (at level 0, right associativity) : bool_scope
V8only.
-Open Scope bool_scope.
+Open Local Scope bool_scope.
(**************************)
(** Lemmas about [negb] *)
diff --git a/theories/ZArith/fast_integer.v b/theories/ZArith/fast_integer.v
index 26a5a738e..7b4e26c03 100644
--- a/theories/ZArith/fast_integer.v
+++ b/theories/ZArith/fast_integer.v
@@ -1313,7 +1313,7 @@ Definition Zcompare := [x,y:Z]
V8Infix "?=" Zcompare (at level 50, no associativity) : Z_scope.
-Open Scope Z_scope.
+Open Local Scope Z_scope.
(**********************************************************************)
(** Properties of opposite on binary integer numbers *)