aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Vectors
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-05-25 12:50:13 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-05-25 12:50:13 +0000
commitbdeccec95e1d018ffb18af9209060a9806d0235a (patch)
treefcc156e3b6ed411cbae70f06e082f07b0b55f4fe /theories/Vectors
parent83e8538118c0b060cb6f231726cda9178f4146bc (diff)
Bugs revealed by playing with contribs
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15364 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Vectors')
-rw-r--r--theories/Vectors/VectorDef.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Vectors/VectorDef.v b/theories/Vectors/VectorDef.v
index 23427eb86..30a8c5699 100644
--- a/theories/Vectors/VectorDef.v
+++ b/theories/Vectors/VectorDef.v
@@ -19,7 +19,7 @@ have to be the same. complain if you see mistakes ... *)
Require Import Arith_base.
Require Vectors.Fin.
Import EqNotations.
-Open Local Scope nat_scope.
+Local Open Scope nat_scope.
(**
A vector is a list of size n whose elements belong to a set A. *)