src/HOL/MicroJava/Comp/TranslCompTp.thy
changeset 80914 d97fdabd9e2b
parent 60773 d09c66a0ea10
--- a/src/HOL/MicroJava/Comp/TranslCompTp.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/MicroJava/Comp/TranslCompTp.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -9,7 +9,7 @@
 (**********************************************************************)
 
 definition comb :: "['a \<Rightarrow> 'b list \<times> 'c, 'c \<Rightarrow> 'b list \<times> 'd, 'a] \<Rightarrow> 'b list \<times> 'd"
-  (infixr "\<box>" 55)
+  (infixr \<open>\<box>\<close> 55)
 where 
   "comb == (\<lambda> f1 f2 x0. let (xs1, x1) = f1 x0; 
                             (xs2, x2) = f2 x1