src/HOLCF/Fun3.thy
changeset 12338 de0f4a63baa5
parent 12030 46d57d0290a2
child 14981 e73f8140af78
--- a/src/HOLCF/Fun3.thy	Sat Dec 01 18:51:46 2001 +0100
+++ b/src/HOLCF/Fun3.thy	Sat Dec 01 18:52:32 2001 +0100
@@ -8,10 +8,10 @@
 
 Fun3 = Fun2 +
 
-(* default class is still term *)
+(* default class is still type *)
 
-instance fun  :: (term,cpo)cpo         (cpo_fun)
-instance fun  :: (term,pcpo)pcpo       (least_fun)
+instance fun  :: (type, cpo) cpo         (cpo_fun)
+instance fun  :: (type, pcpo)pcpo       (least_fun)
 
 end