diff -r 0a01bec9bc13 -r a712bf5ccab0 src/HOL/HOLCF/Cpo.thy --- a/src/HOL/HOLCF/Cpo.thy Wed Dec 11 10:28:12 2024 +0100 +++ b/src/HOL/HOLCF/Cpo.thy Wed Dec 11 10:40:57 2024 +0100 @@ -558,6 +558,7 @@ end + subsection \Discrete cpos\ class discrete_cpo = below + @@ -799,10 +800,12 @@ apply simp done + section \Admissibility and compactness\ default_sort cpo + subsection \Definitions\ definition adm :: "('a::cpo \ bool) \ bool" @@ -969,6 +972,7 @@ adm_below adm_eq adm_not_below adm_compact_not_below adm_compact_neq adm_neq_compact + section \Class instances for the full function space\ subsection \Full function space is a partial order\ @@ -1109,6 +1113,7 @@ for S :: "nat \ 'a::type \ 'b::cpo" by (simp add: lub_fun ch2ch_lambda) + section \The cpo of cartesian products\ subsection \Unit type is a pcpo\ @@ -1401,6 +1406,7 @@ apply (case_tac "\i. Y i", simp) done + section \Discrete cpo types\ datatype 'a discr = Discr "'a :: type"