aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-03 15:01:42 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-03 15:01:42 +0000
commitc88eeed5f7e9c2bfa4eeabba0202659fbd999896 (patch)
treed5eddd04930dd1888abd34b3bf5800434b7d9319 /theories/Init
parentdd12bdb71c15c777d45ebb55f51a3d0bba8f729e (diff)
Essai d'introduction d'un scope des types
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3363 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rw-r--r--theories/Init/DatatypesSyntax.v4
-rwxr-xr-xtheories/Init/Prelude.v2
2 files changed, 4 insertions, 2 deletions
diff --git a/theories/Init/DatatypesSyntax.v b/theories/Init/DatatypesSyntax.v
index 87945b381..52e1328b5 100644
--- a/theories/Init/DatatypesSyntax.v
+++ b/theories/Init/DatatypesSyntax.v
@@ -12,8 +12,8 @@ Require Export Datatypes.
(** Symbolic notations for things in [Datatypes.v] *)
-Infix LEFTA 4 "+" sum.
-Infix RIGHTA 3 "*" prod.
+Infix LEFTA 4 "+" sum : type_scope.
+Infix RIGHTA 3 "*" prod : type_scope.
Notation "( x , y )" := (pair ? ? x y) (at level 0).
Notation Fst := (fst ? ?).
Notation Snd := (snd ? ?).
diff --git a/theories/Init/Prelude.v b/theories/Init/Prelude.v
index 6cdc8d0b4..030ab339e 100755
--- a/theories/Init/Prelude.v
+++ b/theories/Init/Prelude.v
@@ -17,3 +17,5 @@ Require Export SpecifSyntax.
Require Export Peano.
Require Export PeanoSyntax.
Require Export Wf.
+
+Delimits Scope type_scope with T.