src/LCF/lcf.thy
changeset 283 76caebd18756
parent 0 a5a9c433f639
--- a/src/LCF/lcf.thy	Thu Mar 17 13:54:50 1994 +0100
+++ b/src/LCF/lcf.thy	Thu Mar 17 17:48:37 1994 +0100
@@ -12,12 +12,15 @@
 
 default cpo
 
-types tr,void 0
-      "*" 2 (infixl 6)
-      "+" 2 (infixl 5)
+types
+ tr
+ void
+ ('a,'b) "*"		(infixl 6)
+ ('a,'b) "+"		(infixl 5)
 
-arities fun, "*", "+" :: (cpo,cpo)cpo
-        tr,void :: cpo
+arities
+ fun, "*", "+" :: (cpo,cpo)cpo
+ tr,void       :: cpo
 
 consts
  UU	:: "'a"