aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Peano.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 20:53:43 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 20:53:43 +0000
commitd7154b5201733cced13a8e1b3a2e177b98f89eb1 (patch)
tree66e7d88ad1c62e2921ddd287d6031fb6e688dc29 /theories/Init/Peano.v
parentec955042c050eb377fd5d46f95dafb36e5bd7d16 (diff)
nat_scope ouvert par defaut
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4591 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Peano.v')
-rwxr-xr-xtheories/Init/Peano.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Peano.v b/theories/Init/Peano.v
index 077226035..2356c9cb5 100755
--- a/theories/Init/Peano.v
+++ b/theories/Init/Peano.v
@@ -27,7 +27,7 @@ Require Notations.
Require Datatypes.
Require Logic.
-Open Local Scope nat_scope.
+Open Scope nat_scope.
Definition eq_S := (f_equal nat nat S).