aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-05-29 07:36:28 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-05-29 07:36:28 +0000
commit06271582c0227d3c4be9f45c4d8ff408628d9a5c (patch)
tree8e30188f56c036e994d0fab814ed9c6af71a7bc4 /theories/Init/Datatypes.v
parentb49f1fc6d92189a5b9e985042e8d0d07ee0d5220 (diff)
Ajout d'alias pour prodT_rect et cie qui avaient été oublkÃiés
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8872 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Datatypes.v')
-rw-r--r--theories/Init/Datatypes.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index 6ec194325..378b3166e 100644
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -139,6 +139,9 @@ Definition CompOpp (r:comparison) :=
Notation prodT := prod (only parsing).
Notation pairT := pair (only parsing).
+Notation prodT_rect := prod_rect (only parsing).
+Notation prodT_rec := prod_rec (only parsing).
+Notation prodT_ind := prod_ind (only parsing).
Notation fstT := fst (only parsing).
Notation sndT := snd (only parsing).
Notation prodT_uncurry := prod_uncurry (only parsing).