src/HOL/HOLCF/Cpodef.thy
changeset 81575 cb57350beaa9
parent 69913 ca515cf61651
child 81584 a065d8bcfd3d
--- a/src/HOL/HOLCF/Cpodef.thy	Tue Dec 10 22:40:07 2024 +0100
+++ b/src/HOL/HOLCF/Cpodef.thy	Tue Dec 10 22:59:13 2024 +0100
@@ -5,7 +5,7 @@
 section \<open>Subtypes of pcpos\<close>
 
 theory Cpodef
-  imports Adm
+  imports Cpo
   keywords "pcpodef" "cpodef" :: thy_goal_defn
 begin
 
@@ -16,7 +16,7 @@
   if the ordering is defined in the standard way.
 \<close>
 
-setup \<open>Sign.add_const_constraint (\<^const_name>\<open>Porder.below\<close>, NONE)\<close>
+setup \<open>Sign.add_const_constraint (\<^const_name>\<open>below\<close>, NONE)\<close>
 
 theorem typedef_po:
   fixes Abs :: "'a::po \<Rightarrow> 'b::type"
@@ -30,7 +30,7 @@
   apply (erule (1) below_antisym)
   done
 
-setup \<open>Sign.add_const_constraint (\<^const_name>\<open>Porder.below\<close>, SOME \<^typ>\<open>'a::below \<Rightarrow> 'a::below \<Rightarrow> bool\<close>)\<close>
+setup \<open>Sign.add_const_constraint (\<^const_name>\<open>below\<close>, SOME \<^typ>\<open>'a::below \<Rightarrow> 'a::below \<Rightarrow> bool\<close>)\<close>
 
 
 subsection \<open>Proving a subtype is finite\<close>