--- a/src/HOL/HOLCF/Lift.thy Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/HOLCF/Lift.thy Fri Sep 20 19:51:08 2024 +0200
@@ -85,7 +85,7 @@
subsection \<open>Further operations\<close>
definition
- flift1 :: "('a \<Rightarrow> 'b::pcpo) \<Rightarrow> ('a lift \<rightarrow> 'b)" (binder "FLIFT " 10) where
+ flift1 :: "('a \<Rightarrow> 'b::pcpo) \<Rightarrow> ('a lift \<rightarrow> 'b)" (binder \<open>FLIFT \<close> 10) where
"flift1 = (\<lambda>f. (\<Lambda> x. case_lift \<bottom> f x))"
translations