summaryrefslogtreecommitdiff
path: root/theories/Init/Logic_Type.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Init/Logic_Type.v')
-rw-r--r--theories/Init/Logic_Type.v28
1 files changed, 1 insertions, 27 deletions
diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v
index 857ffe94..dbe944b0 100644
--- a/theories/Init/Logic_Type.v
+++ b/theories/Init/Logic_Type.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id: Logic_Type.v 8642 2006-03-17 10:09:02Z notin $ i*)
+(*i $Id: Logic_Type.v 8866 2006-05-28 16:21:04Z herbelin $ i*)
(** This module defines type constructors for types in [Type]
([Datatypes.v] and [Logic.v] defined them for types in [Set]) *)
@@ -20,32 +20,6 @@ Require Export Logic.
Definition notT (A:Type) := A -> False.
-(** Conjunction of types in [Type] *)
-
-Inductive prodT (A B:Type) : Type :=
- pairT : A -> B -> prodT A B.
-
-Section prodT_proj.
-
- Variables A B : Type.
-
- Definition fstT (H:prodT A B) := match H with
- | pairT x _ => x
- end.
- Definition sndT (H:prodT A B) := match H with
- | pairT _ y => y
- end.
-
-End prodT_proj.
-
-Definition prodT_uncurry (A B C:Type) (f:prodT A B -> C)
- (x:A) (y:B) : C := f (pairT x y).
-
-Definition prodT_curry (A B C:Type) (f:A -> B -> C)
- (p:prodT A B) : C := match p with
- | pairT x y => f x y
- end.
-
(** Properties of [identity] *)
Section identity_is_a_congruence.