aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic_Type.v
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-05-15 07:47:00 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-05-15 07:47:00 +0000
commitd2510f9a76cef997e22e1968031c5317be2b7c8f (patch)
treefbcf25ebbcaac1e83082a838f34829013954bf23 /theories/Init/Logic_Type.v
parent675884d2e03507602f4149eec7917d047b82e941 (diff)
Modification pour passage p-automates
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1753 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Logic_Type.v')
-rwxr-xr-xtheories/Init/Logic_Type.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v
index 35a25a46f..81805c9c4 100755
--- a/theories/Init/Logic_Type.v
+++ b/theories/Init/Logic_Type.v
@@ -211,7 +211,10 @@ 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].