src/HOL/HOLCF/Cfun.thy
changeset 81583 b6df83045178
parent 81575 cb57350beaa9
child 81946 ee680c69de38
--- a/src/HOL/HOLCF/Cfun.thy	Thu Dec 12 12:35:59 2024 +0100
+++ b/src/HOL/HOLCF/Cfun.thy	Thu Dec 12 15:45:29 2024 +0100
@@ -9,9 +9,6 @@
   imports Cpodef
 begin
 
-default_sort cpo
-
-
 subsection \<open>Definition of continuous function type\<close>
 
 definition "cfun = {f::'a \<Rightarrow> 'b. cont f}"
@@ -455,9 +452,7 @@
 
 subsection \<open>Strictified functions\<close>
 
-default_sort pcpo
-
-definition seq :: "'a \<rightarrow> 'b \<rightarrow> 'b"
+definition seq :: "'a::pcpo \<rightarrow> 'b::pcpo \<rightarrow> 'b"
   where "seq = (\<Lambda> x. if x = \<bottom> then \<bottom> else ID)"
 
 lemma cont2cont_if_bottom [cont2cont, simp]:
@@ -481,7 +476,7 @@
   "x \<noteq> \<bottom> \<Longrightarrow> seq\<cdot>x = ID"
   by (simp_all add: seq_conv_if)
 
-definition strictify  :: "('a \<rightarrow> 'b) \<rightarrow> 'a \<rightarrow> 'b"
+definition strictify  :: "('a::pcpo \<rightarrow> 'b::pcpo) \<rightarrow> 'a \<rightarrow> 'b"
   where "strictify = (\<Lambda> f x. seq\<cdot>x\<cdot>(f\<cdot>x))"
 
 lemma strictify_conv_if: "strictify\<cdot>f\<cdot>x = (if x = \<bottom> then \<bottom> else f\<cdot>x)"