--- a/src/HOL/Examples/Adhoc_Overloading_Examples.thy Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Examples/Adhoc_Overloading_Examples.thy Fri Sep 20 19:51:08 2024 +0200
@@ -176,7 +176,7 @@
this end we introduce a constant \<open>PERMUTE\<close> together with
convenient infix syntax.\<close>
-consts PERMUTE :: "'a perm \<Rightarrow> 'b \<Rightarrow> 'b" (infixr "\<bullet>" 75)
+consts PERMUTE :: "'a perm \<Rightarrow> 'b \<Rightarrow> 'b" (infixr \<open>\<bullet>\<close> 75)
text \<open>Then we add a locale for types \<^typ>\<open>'b\<close> that support
appliciation of permutations.\<close>