src/HOLCF/Ssum0.thy
changeset 1150 66512c9e6bd6
parent 243 c22b85994e17
child 1168 74be52691d62
--- a/src/HOLCF/Ssum0.thy	Wed Jun 21 15:01:07 1995 +0200
+++ b/src/HOLCF/Ssum0.thy	Wed Jun 21 15:14:58 1995 +0200
@@ -26,11 +26,11 @@
 
 rules
 
-  Sinl_Rep_def		"Sinl_Rep == (%a.%x y p.\
-\				(~a=UU --> x=a  & p))"
+  Sinl_Rep_def		"Sinl_Rep == (%a.%x y p.
+				(~a=UU --> x=a  & p))"
 
-  Sinr_Rep_def		"Sinr_Rep == (%b.%x y p.\
-\				(~b=UU --> y=b  & ~p))"
+  Sinr_Rep_def		"Sinr_Rep == (%b.%x y p.
+				(~b=UU --> y=b  & ~p))"
 
   Ssum_def		"Ssum =={f.(? a.f=Sinl_Rep(a))|(? b.f=Sinr_Rep(b))}"
 
@@ -45,10 +45,10 @@
   Isinl_def	"Isinl(a) == Abs_Ssum(Sinl_Rep(a))"
   Isinr_def	"Isinr(b) == Abs_Ssum(Sinr_Rep(b))"
 
-  Iwhen_def	"Iwhen(f)(g)(s) == @z.\
-\				    (s=Isinl(UU) --> z=UU)\
-\			&(!a. ~a=UU & s=Isinl(a) --> z=f[a])\  
-\			&(!b. ~b=UU & s=Isinr(b) --> z=g[b])"  
+  Iwhen_def	"Iwhen(f)(g)(s) == @z.
+				    (s=Isinl(UU) --> z=UU)
+			&(!a. ~a=UU & s=Isinl(a) --> z=f[a])
+			&(!b. ~b=UU & s=Isinr(b) --> z=g[b])"  
 
 end