src/HOLCF/Cfun.thy
changeset 40091 1ca61fbd8a79
parent 40089 8adc57fb8454
child 40093 c2d36bc4cd14
--- a/src/HOLCF/Cfun.thy	Fri Oct 22 07:44:34 2010 -0700
+++ b/src/HOLCF/Cfun.thy	Fri Oct 22 07:45:32 2010 -0700
@@ -95,9 +95,6 @@
 lemma UU_CFun: "\<bottom> \<in> CFun"
 by (simp add: CFun_def inst_fun_pcpo)
 
-instance cfun :: ("{finite,cpo}", chfin) chfin
-by (rule typedef_chfin [OF type_definition_CFun below_CFun_def])
-
 instance cfun :: (cpo, discrete_cpo) discrete_cpo
 by intro_classes (simp add: below_CFun_def Rep_CFun_inject)