diff -r 6023808b38d4 -r 1c6f7d4b110e src/HOLCF/Up.thy --- a/src/HOLCF/Up.thy Sat Nov 27 12:55:12 2010 -0800 +++ b/src/HOLCF/Up.thy Sat Nov 27 13:12:10 2010 -0800 @@ -111,7 +111,7 @@ proof (rule up_chain_lemma) assume "\i. S i = Ibottom" hence "range (\i. S i) <<| Ibottom" - by (simp add: lub_const) + by (simp add: is_lub_const) thus ?thesis .. next fix A :: "nat \ 'a" @@ -160,7 +160,7 @@ assume A: "\i. Iup (A i) = Y (i + k)" assume "chain A" and "range Y <<| Iup (\i. A i)" hence "Ifup f (\i. Y i) = (\i. Ifup f (Iup (A i)))" - by (simp add: thelubI contlub_cfun_arg) + by (simp add: lub_eqI contlub_cfun_arg) also have "\ = (\i. Ifup f (Y (i + k)))" by (simp add: A) also have "\ = (\i. Ifup f (Y i))" @@ -223,7 +223,7 @@ assumes Y: "chain Y" obtains "\i. Y i = \" | A k where "\i. up\(A i) = Y (i + k)" and "chain A" and "(\i. Y i) = up\(\i. A i)" apply (rule up_chain_lemma [OF Y]) -apply (simp_all add: inst_up_pcpo up_def cont_Iup thelubI) +apply (simp_all add: inst_up_pcpo up_def cont_Iup lub_eqI) done lemma compact_up: "compact x \ compact (up\x)"