add lemma ub2ub_monofun'
authorhuffman
Wed, 02 Jan 2008 18:28:15 +0100
changeset 25783 b2874ee9081a
parent 25782 2d8b845dc298
child 25784 71157f7e671e
add lemma ub2ub_monofun'
src/HOLCF/Cont.thy
--- a/src/HOLCF/Cont.thy	Wed Jan 02 18:27:07 2008 +0100
+++ b/src/HOLCF/Cont.thy	Wed Jan 02 18:28:15 2008 +0100
@@ -89,6 +89,13 @@
 apply (erule ub_rangeD)
 done
 
+lemma ub2ub_monofun':
+  "\<lbrakk>monofun f; S <| u\<rbrakk> \<Longrightarrow> f ` S <| f u"
+apply (rule ub_imageI)
+apply (erule monofunE)
+apply (erule (1) is_ubD)
+done
+
 text {* monotone functions map directed sets to directed sets *}
 
 lemma dir2dir_monofun: