src/HOLCF/Cfun2.thy
changeset 1479 21eb5e156d91
parent 1168 74be52691d62
child 2640 ee4dfce170a0
--- a/src/HOLCF/Cfun2.thy	Tue Feb 06 12:27:17 1996 +0100
+++ b/src/HOLCF/Cfun2.thy	Tue Feb 06 12:42:31 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	HOLCF/cfun2.thy
+(*  Title:      HOLCF/cfun2.thy
     ID:         $Id$
-    Author: 	Franz Regensburger
+    Author:     Franz Regensburger
     Copyright   1993 Technische Universitaet Muenchen
 
 Class Instance ->::(pcpo,pcpo)po
@@ -12,19 +12,19 @@
 (* Witness for the above arity axiom is cfun1.ML *)
 arities "->" :: (pcpo,pcpo)po
 
-consts	
-	UU_cfun  :: "'a->'b"
+consts  
+        UU_cfun  :: "'a->'b"
 
 rules
 
 (* instance of << for type ['a -> 'b]  *)
 
-inst_cfun_po	"((op <<)::['a->'b,'a->'b]=>bool) = less_cfun"
+inst_cfun_po    "((op <<)::['a->'b,'a->'b]=>bool) = less_cfun"
 
 defs
 (* The least element in type 'a->'b *)
 
-UU_cfun_def	"UU_cfun == fabs(% x.UU)"
+UU_cfun_def     "UU_cfun == fabs(% x.UU)"
 
 end