src/HOLCF/Fun3.thy
changeset 15564 c899efea601f
parent 14981 e73f8140af78
--- a/src/HOLCF/Fun3.thy	Wed Mar 02 22:57:08 2005 +0100
+++ b/src/HOLCF/Fun3.thy	Wed Mar 02 23:15:16 2005 +0100
@@ -1,16 +1,35 @@
 (*  Title:      HOLCF/Fun3.thy
     ID:         $Id$
     Author:     Franz Regensburger
+    License:    GPL (GNU GENERAL PUBLIC LICENSE)
 
 Class instance of  => (fun) for class pcpo
 *)
 
-Fun3 = Fun2 +
+theory Fun3 = Fun2:
 
 (* default class is still type *)
 
-instance fun  :: (type, cpo) cpo         (cpo_fun)
-instance fun  :: (type, pcpo)pcpo       (least_fun)
+instance fun  :: (type, cpo) cpo
+apply (intro_classes)
+apply (erule cpo_fun)
+done
+
+instance fun  :: (type, pcpo)pcpo
+apply (intro_classes)
+apply (rule least_fun)
+done
+
+(*  Title:      HOLCF/Fun3.ML
+    ID:         $Id$
+    Author:     Franz Regensburger
+    License:    GPL (GNU GENERAL PUBLIC LICENSE)
+*)
+
+(* for compatibility with old HOLCF-Version *)
+lemma inst_fun_pcpo: "UU = (%x. UU)"
+apply (simp add: UU_def UU_fun_def)
+done
 
 end