src/HOL/Sum.thy
changeset 1370 7361ac9b024d
parent 1151 c820b3cc3df0
child 1423 5726a8243d3f
--- a/src/HOL/Sum.thy	Mon Nov 27 13:44:56 1995 +0100
+++ b/src/HOL/Sum.thy	Wed Nov 29 16:44:59 1995 +0100
@@ -11,8 +11,8 @@
 (* type definition *)
 
 consts
-  Inl_Rep       :: "['a, 'a, 'b, bool] => bool"
-  Inr_Rep       :: "['b, 'a, 'b, bool] => bool"
+  Inl_Rep       :: ['a, 'a, 'b, bool] => bool
+  Inr_Rep       :: ['b, 'a, 'b, bool] => bool
 
 defs
   Inl_Rep_def   "Inl_Rep == (%a. %x y p. x=a & p)"
@@ -32,7 +32,7 @@
 
   (*disjoint sum for sets; the operator + is overloaded with wrong type!*)
   "plus"        :: "['a set, 'b set] => ('a + 'b) set"        (infixr 65)
-  Part          :: "['a set, 'b => 'a] => 'a set"
+  Part          :: ['a set, 'b => 'a] => 'a set
 
 translations
   "case p of Inl(x) => a | Inr(y) => b" == "sum_case (%x.a) (%y.b) p"