aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Notations.v
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/Init/Notations.v
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/Init/Notations.v')
-rw-r--r--theories/Init/Notations.v10
1 files changed, 1 insertions, 9 deletions
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 *)