From bdeccec95e1d018ffb18af9209060a9806d0235a Mon Sep 17 00:00:00 2001 From: pboutill Date: Fri, 25 May 2012 12:50:13 +0000 Subject: Bugs revealed by playing with contribs git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15364 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Vectors/VectorDef.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Vectors') 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. *) -- cgit v1.2.3