aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zminmax.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-02-12 22:08:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-02-12 22:08:04 +0000
commit9ff6f3029e0a275d8630f055bdb78e2c15e8bb29 (patch)
tree72f20a199ed91db9a1923f836a0fc2f5681bb569 /theories/ZArith/Zminmax.v
parent6ac0fe66443ceff379223ab3581806fa1fced987 (diff)
Bug Scope
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8034 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zminmax.v')
-rw-r--r--theories/ZArith/Zminmax.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zminmax.v b/theories/ZArith/Zminmax.v
index c311c7ce9..a862c5619 100644
--- a/theories/ZArith/Zminmax.v
+++ b/theories/ZArith/Zminmax.v
@@ -10,7 +10,7 @@
Require Import Zmin Zmax.
Require Import BinInt Zorder.
-Open Scope Z_scope.
+Open Local Scope Z_scope.
(** *** Lattice properties of min and max on Z *)