aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
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.