src/HOLCF/Cont.thy
changeset 25825 94c075b912ff
parent 25786 6b3c79acac1f
child 25896 b2d2f1ae5808
--- 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)