src/HOL/SMT_Examples/Boogie.thy
changeset 80914 d97fdabd9e2b
parent 72741 b808eddc83cf
--- a/src/HOL/SMT_Examples/Boogie.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/SMT_Examples/Boogie.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -38,8 +38,8 @@
 \<close>
 
 axiomatization
-  boogie_div :: "int \<Rightarrow> int \<Rightarrow> int" (infixl "div'_b" 70) and
-  boogie_mod :: "int \<Rightarrow> int \<Rightarrow> int" (infixl "mod'_b" 70)
+  boogie_div :: "int \<Rightarrow> int \<Rightarrow> int" (infixl \<open>div'_b\<close> 70) and
+  boogie_mod :: "int \<Rightarrow> int \<Rightarrow> int" (infixl \<open>mod'_b\<close> 70)