src/HOLCF/Adm.thy
changeset 25786 6b3c79acac1f
parent 25131 2c8caac48ade
child 25802 8aea40e25aa8
--- a/src/HOLCF/Adm.thy	Wed Jan 02 18:54:21 2008 +0100
+++ b/src/HOLCF/Adm.thy	Wed Jan 02 18:57:40 2008 +0100
@@ -140,6 +140,8 @@
 
 text {* admissibility and continuity *}
 
+declare range_composition [simp del]
+
 lemma adm_less: "\<lbrakk>cont u; cont v\<rbrakk> \<Longrightarrow> adm (\<lambda>x. u x \<sqsubseteq> v x)"
 apply (rule admI)
 apply (simp add: cont2contlubE)
@@ -165,7 +167,7 @@
 apply (drule_tac x=0 in spec)
 apply (erule contrapos_nn)
 apply (erule rev_trans_less)
-apply (erule cont2mono [THEN monofun_fun_arg])
+apply (erule cont2mono [THEN monofunE])
 apply (erule is_ub_thelub)
 done