generalized chfindom_monofun2cont
authorhuffman
Thu, 03 Jan 2008 23:58:27 +0100
changeset 25825 94c075b912ff
parent 25824 f56dd9745d1b
child 25826 f9aa43287e42
generalized chfindom_monofun2cont
src/HOLCF/Cont.thy
--- a/src/HOLCF/Cont.thy	Thu Jan 03 23:19:30 2008 +0100
+++ b/src/HOLCF/Cont.thy	Thu Jan 03 23:58:27 2008 +0100
@@ -189,7 +189,7 @@
   "\<lbrakk>cont f; finite_chain Y\<rbrakk> \<Longrightarrow> finite_chain (\<lambda>n. f (Y n))"
 by (rule cont2mono [THEN monofun_finch2finch])
 
-lemma chfindom_monofun2cont: "monofun f \<Longrightarrow> cont (f::'a::chfin \<Rightarrow> 'b::pcpo)"
+lemma chfindom_monofun2cont: "monofun f \<Longrightarrow> cont (f::'a::chfin \<Rightarrow> 'b::cpo)"
 apply (rule monocontlub2cont)
 apply assumption
 apply (rule contlubI)