src/HOLCF/fun2.thy
changeset 13897 f62f9a75f685
parent 13896 717bd79b976f
child 13898 9410d2eb9563
--- a/src/HOLCF/fun2.thy	Sat Apr 05 17:03:38 2003 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,40 +0,0 @@
-(*  Title: 	HOLCF/fun2.thy
-    ID:         $Id$
-    Author: 	Franz Regensburger
-    Copyright   1993 Technische Universitaet Muenchen
-
-Class Instance =>::(term,po)po
-Definiton of least element
-*)
-
-Fun2 = Fun1 + 
-
-(* default class is still term !*)
-
-(* Witness for the above arity axiom is fun1.ML *)
-
-arities fun :: (term,po)po
-
-consts	
-	UU_fun  :: "'a::term => 'b::pcpo"
-
-rules
-
-(* instance of << for type ['a::term => 'b::po]  *)
-
-inst_fun_po	"(op <<)::['a=>'b::po,'a=>'b::po ]=>bool = less_fun"
-
-(* definitions *)
-(* The least element in type 'a::term => 'b::pcpo *)
-
-UU_fun_def	"UU_fun == (% x.UU)"
-
-end
-
-
-
-
-
-
-
-