src/HOLCF/Fun_Cpo.thy
changeset 40004 9f6ed6840e8d
parent 40002 c5b5f7a3a3b1
child 40006 116e94f9543b
--- a/src/HOLCF/Fun_Cpo.thy	Tue Oct 12 05:25:21 2010 -0700
+++ b/src/HOLCF/Fun_Cpo.thy	Tue Oct 12 05:48:15 2010 -0700
@@ -204,10 +204,6 @@
 apply (simp add: diag_lub ch2ch_fun ch2ch_cont)
 done
 
-lemma cont2cont_lub:
-  "\<lbrakk>chain F; \<And>i. cont (F i)\<rbrakk> \<Longrightarrow> cont (\<lambda>x. \<Squnion>i. F i x)"
-by (simp add: thelub_fun [symmetric] cont_lub_fun)
-
 lemma mono2mono_fun: "monofun f \<Longrightarrow> monofun (\<lambda>x. f x y)"
 apply (rule monofunI)
 apply (erule (1) monofun_fun_arg [THEN monofun_fun_fun])