aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic_Type.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-11-24 23:12:49 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-11-24 23:12:49 +0000
commitd2b7a94fe0ed982a6dd7ff2c07991c2f1b1a6fc8 (patch)
tree8a1fb9004b2eaa86621089b901f495688bfc6990 /theories/Init/Logic_Type.v
parentde7212f0fe40d7b83748f9d4473311b9884d93fa (diff)
Généralisation de l'utilisation de Notation
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3269 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Logic_Type.v')
-rwxr-xr-xtheories/Init/Logic_Type.v4
1 files changed, 0 insertions, 4 deletions
diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v
index 80cd878b1..e4982c1f6 100755
--- a/theories/Init/Logic_Type.v
+++ b/theories/Init/Logic_Type.v
@@ -198,10 +198,6 @@ Definition prodT_curry : (A,B,C:Type)(A->B->C)->(prodT A B)->C :=
Hints Immediate sym_idT sym_not_idT : core v62.
-Syntactic Definition AllT := allT | 1.
-Syntactic Definition ExT := exT | 1.
-Syntactic Definition ExT2 := exT2 | 1.
-
Implicits fstT [1 2].
Implicits sndT [1 2].
Implicits pairT [1 2].