src/HOL/HOLCF/Up.thy
changeset 80914 d97fdabd9e2b
parent 69597 ff784d5a5bfb
child 81095 49c04500c5f9
--- a/src/HOL/HOLCF/Up.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/HOLCF/Up.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -14,7 +14,7 @@
 
 subsection \<open>Definition of new type for lifting\<close>
 
-datatype 'a u  ("(_\<^sub>\<bottom>)" [1000] 999) = Ibottom | Iup 'a
+datatype 'a u  (\<open>(_\<^sub>\<bottom>)\<close> [1000] 999) = Ibottom | Iup 'a
 
 primrec Ifup :: "('a \<rightarrow> 'b::pcpo) \<Rightarrow> 'a u \<Rightarrow> 'b"
   where