changeset 40002 | c5b5f7a3a3b1 |
parent 39984 | 0300d5170622 |
child 40500 | ee9c8d36318e |
--- a/src/HOLCF/Completion.thy Mon Oct 11 16:24:44 2010 -0700 +++ b/src/HOLCF/Completion.thy Mon Oct 11 21:35:31 2010 -0700 @@ -397,7 +397,7 @@ assumes g_mono: "\<And>a b. a \<preceq> b \<Longrightarrow> g a \<sqsubseteq> g b" assumes below: "\<And>a. f a \<sqsubseteq> g a" shows "basis_fun f \<sqsubseteq> basis_fun g" - apply (rule below_cfun_ext) + apply (rule cfun_belowI) apply (simp only: basis_fun_beta f_mono g_mono) apply (rule is_lub_thelub_ex) apply (rule basis_fun_lemma, erule f_mono)