src/HOLCF/cfun3.thy
changeset 13897 f62f9a75f685
parent 13896 717bd79b976f
child 13898 9410d2eb9563
--- a/src/HOLCF/cfun3.thy	Sat Apr 05 17:03:38 2003 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,31 +0,0 @@
-(*  Title: 	HOLCF/cfun3.thy
-    ID:         $Id$
-    Author: 	Franz Regensburger
-    Copyright   1993 Technische Universitaet Muenchen
-
-Class instance of  -> for class pcpo
-
-*)
-
-Cfun3 = Cfun2 +
-
-arities "->"	:: (pcpo,pcpo)pcpo		(* Witness cfun2.ML *)
-
-consts  
-	Istrictify   :: "('a->'b)=>'a=>'b"
-	strictify    :: "('a->'b)->'a->'b"
-
-rules 
-
-inst_cfun_pcpo	"UU::'a->'b = UU_cfun"
-
-Istrictify_def	"Istrictify(f,x) == (@z.\
-\			  ( x=UU --> z = UU)\
-\			& (~x=UU --> z = f[x]))"	
-
-strictify_def	"strictify == (LAM f x.Istrictify(f,x))"
-
-end
-
-
-