aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-03-17 10:54:50 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-03-17 10:54:50 +0000
commit4745361bce67612914052afcd3a05d1636ddb97e (patch)
treeed5fdb7f805ec44c5c98b0073fb17cfebb81829d /theories
parentfe0a1f5e856b702a5e4638e22b748d2d8af475c2 (diff)
Definition de la notation de la paire par un motif recursif
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5518 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rwxr-xr-xtheories/Init/Datatypes.v13
-rw-r--r--theories/Init/Notations.v10
2 files changed, 2 insertions, 21 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index 7c199bbf3..353ba073e 100755
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -77,18 +77,7 @@ Inductive prod (A B:Set) : Set :=
Add Printing Let prod.
Notation "x * y" := (prod x y) : type_scope.
-Notation "( x , y )" := (pair x y) : core_scope.
-
-(* Temporary hack *)
-Notation "( x1 , x2 , x3 )" := ((x1,x2),x3) : core_scope.
-Notation "( x1 , x2 , x3 , x4 )" := ((x1,x2),x3,x4) : core_scope.
-Notation "( x1 , x2 , x3 , x4 , x5 )" := ((x1,x2),x3,x4,x5) : core_scope.
-Notation "( x1 , x2 , x3 , x4 , x5 , x6 )"
- := ((x1,x2),x3,x4,x5,x6) : core_scope.
-Notation "( x1 , x2 , x3 , x4 , x5 , x6 , x7 )"
- := ((x1,x2),x3,x4,x5,x6,x7) : core_scope.
-Notation "( x1 , x2 , x3 , x4 , x5 , x6 , x7 , x8 )"
- := ((x1,x2),x3,x4,x5,x6,x7,x8) : core_scope.
+Notation "( x , y , .. , z )" := (pair .. (pair x y) .. z) : core_scope.
Section projections.
Variables A B : Set.
diff --git a/theories/Init/Notations.v b/theories/Init/Notations.v
index 92e1a818b..791500986 100644
--- a/theories/Init/Notations.v
+++ b/theories/Init/Notations.v
@@ -51,15 +51,7 @@ Reserved Notation "x ^ y" (at level 30, right associativity).
(** Notations for pairs *)
-(* Temporary hack *)
-Reserved Notation "( x , y )" (at level 0).
-Reserved Notation "( x , y , z )" (at level 0).
-Reserved Notation "( x1 , x2 , x3 )" (at level 0).
-Reserved Notation "( x1 , x2 , x3 , x4 )" (at level 0).
-Reserved Notation "( x1 , x2 , x3 , x4 , x5 )" (at level 0).
-Reserved Notation "( x1 , x2 , x3 , x4 , x5 , x6 )" (at level 0).
-Reserved Notation "( x1 , x2 , x3 , x4 , x5 , x6 , x7 )" (at level 0).
-Reserved Notation "( x1 , x2 , x3 , x4 , x5 , x6 , x7 , x8 )" (at level 0).
+Reserved Notation "( x , y , .. , z )" (at level 0).
(** Notation "{ x }" is reserved and has a special status as component
of other notations; it is at level 0 to factor with {x:A|P} etc *)