src/HOLCF/Pcpo.thy
changeset 1479 21eb5e156d91
parent 1274 ea0668a1c0ba
child 2278 d63ffafce255
--- a/src/HOLCF/Pcpo.thy	Tue Feb 06 12:27:17 1996 +0100
+++ b/src/HOLCF/Pcpo.thy	Tue Feb 06 12:42:31 1996 +0100
@@ -3,15 +3,15 @@
 classes pcpo < po
 arities void :: pcpo
 
-consts	
-	UU :: "'a::pcpo"	
+consts  
+        UU :: "'a::pcpo"        
 
 rules
 
-	minimal	"UU << x"	
-	cpo	"is_chain(S) ==> ? x. range(S) <<| (x::'a::pcpo)" 
+        minimal "UU << x"       
+        cpo     "is_chain(S) ==> ? x. range(S) <<| (x::'a::pcpo)" 
 
-inst_void_pcpo	"(UU::void) = UU_void"
+inst_void_pcpo  "(UU::void) = UU_void"
 
 (* start 8bit 1 *)
 (* end 8bit 1 *)