src/HOL/HOLCF/Pcpo.thy
changeset 80914 d97fdabd9e2b
parent 80768 c7723cc15de8
child 81101 8407b4c068e2
--- a/src/HOL/HOLCF/Pcpo.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/HOLCF/Pcpo.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -136,7 +136,7 @@
   assumes least: "\<exists>x. \<forall>y. x \<sqsubseteq> y"
 begin
 
-definition bottom :: "'a"  ("\<bottom>")
+definition bottom :: "'a"  (\<open>\<bottom>\<close>)
   where "bottom = (THE x. \<forall>y. x \<sqsubseteq> y)"
 
 lemma minimal [iff]: "\<bottom> \<sqsubseteq> x"