src/HOL/Univ.thy
changeset 5978 fa2c2dd74f8c
parent 5191 8ceaa19f7717
child 7014 11ee650edcd2
--- a/src/HOL/Univ.thy	Thu Nov 26 17:40:10 1998 +0100
+++ b/src/HOL/Univ.thy	Fri Nov 27 10:40:29 1998 +0100
@@ -42,7 +42,6 @@
   Split  :: [['a item, 'a item]=>'b, 'a item] => 'b
   Case   :: [['a item]=>'b, ['a item]=>'b, 'a item] => 'b
 
-  diag   :: "'a set => ('a * 'a)set"
   "<**>" :: "[('a item * 'a item)set, ('a item * 'a item)set] 
            => ('a item * 'a item)set" (infixr 80)
   "<++>" :: "[('a item * 'a item)set, ('a item * 'a item)set] 
@@ -88,13 +87,11 @@
                               | (? y . M = In1(y) & u = d(y))"
 
 
-  (** diagonal sets and equality for the "universe" **)
-
-  diag_def   "diag(A) == UN x:A. {(x,x)}"
+  (** equality for the "universe" **)
 
   dprod_def  "r<**>s == UN (x,x'):r. UN (y,y'):s. {(Scons x y, Scons x' y')}"
 
   dsum_def   "r<++>s == (UN (x,x'):r. {(In0(x),In0(x'))}) Un 
-                       (UN (y,y'):s. {(In1(y),In1(y'))})"
+                        (UN (y,y'):s. {(In1(y),In1(y'))})"
 
 end