diff -r 0a01bec9bc13 -r a712bf5ccab0 src/HOL/HOLCF/Lift.thy --- a/src/HOL/HOLCF/Lift.thy Wed Dec 11 10:28:12 2024 +0100 +++ b/src/HOL/HOLCF/Lift.thy Wed Dec 11 10:40:57 2024 +0100 @@ -19,6 +19,7 @@ Def :: "'a \ 'a lift" where "Def x = Abs_lift (up\(Discr x))" + subsection \Lift as a datatype\ lemma lift_induct: "\P \; \x. P (Def x)\ \ P y" @@ -70,6 +71,7 @@ by (induct x) auto qed + subsection \Continuity of \<^const>\case_lift\\ lemma case_lift_eq: "case_lift \ f x = fup\(\ y. f (undiscr y))\(Rep_lift x)" @@ -82,6 +84,7 @@ "\\y. cont (\x. f x y); cont g\ \ cont (\x. case_lift \ (f x) (g x))" unfolding case_lift_eq by (simp add: cont_Rep_lift) + subsection \Further operations\ definition