src/HOL/IMP/Def_Init_Big.thy
changeset 80914 d97fdabd9e2b
parent 69597 ff784d5a5bfb
--- a/src/HOL/IMP/Def_Init_Big.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/IMP/Def_Init_Big.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -7,7 +7,7 @@
 subsection "Initialization-Sensitive Big Step Semantics"
 
 inductive
-  big_step :: "(com \<times> state option) \<Rightarrow> state option \<Rightarrow> bool" (infix "\<Rightarrow>" 55)
+  big_step :: "(com \<times> state option) \<Rightarrow> state option \<Rightarrow> bool" (infix \<open>\<Rightarrow>\<close> 55)
 where
 None: "(c,None) \<Rightarrow> None" |
 Skip: "(SKIP,s) \<Rightarrow> s" |