new lemma cont_discrete_cpo
authorhuffman
Thu, 31 Jan 2008 21:22:03 +0100
changeset 26024 d5129e687290
parent 26023 29c1e3e98276
child 26025 ca6876116bb4
new lemma cont_discrete_cpo
src/HOLCF/Cont.thy
--- a/src/HOLCF/Cont.thy	Thu Jan 31 21:21:22 2008 +0100
+++ b/src/HOLCF/Cont.thy	Thu Jan 31 21:22:03 2008 +0100
@@ -229,4 +229,12 @@
 lemma flatdom_strict2cont: "f \<bottom> = \<bottom> \<Longrightarrow> cont (f::'a::flat \<Rightarrow> 'b::pcpo)"
 by (rule flatdom_strict2mono [THEN chfindom_monofun2cont])
 
+text {* functions with discrete domain *}
+
+lemma cont_discrete_cpo [simp]: "cont (f::'a::discrete_cpo \<Rightarrow> 'b::cpo)"
+apply (rule contI)
+apply (drule discrete_chain_const, clarify)
+apply (simp add: lub_const)
+done
+
 end