src/HOLCF/Cfun.thy
changeset 25901 bb178c8251e0
parent 25884 a69e665b7df8
child 25920 8df5eabda5f6
equal deleted inserted replaced
25900:464f23aa905f 25901:bb178c8251e0
   249     \<Longrightarrow> (\<Lambda> x. \<Squnion>i. F i x) = (\<Squnion>i. \<Lambda> x. F i x)"
   249     \<Longrightarrow> (\<Lambda> x. \<Squnion>i. F i x) = (\<Squnion>i. \<Lambda> x. F i x)"
   250 apply (simp add: thelub_CFun)
   250 apply (simp add: thelub_CFun)
   251 apply (simp add: Abs_CFun_inverse2)
   251 apply (simp add: Abs_CFun_inverse2)
   252 apply (simp add: thelub_fun ch2ch_lambda)
   252 apply (simp add: thelub_fun ch2ch_lambda)
   253 done
   253 done
       
   254 
       
   255 lemmas lub_distribs = 
       
   256   contlub_cfun [symmetric]
       
   257   contlub_LAM [symmetric]
   254 
   258 
   255 text {* strictness *}
   259 text {* strictness *}
   256 
   260 
   257 lemma strictI: "f\<cdot>x = \<bottom> \<Longrightarrow> f\<cdot>\<bottom> = \<bottom>"
   261 lemma strictI: "f\<cdot>x = \<bottom> \<Longrightarrow> f\<cdot>\<bottom> = \<bottom>"
   258 apply (rule UU_I)
   262 apply (rule UU_I)