src/HOL/Bali/State.thy
changeset 80914 d97fdabd9e2b
parent 80768 c7723cc15de8
child 81278 41e843d901ee
--- a/src/HOL/Bali/State.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Bali/State.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -183,7 +183,7 @@
 done
 
 definition
-  in_bounds :: "int \<Rightarrow> int \<Rightarrow> bool" ("(_/ in'_bounds _)" [50, 51] 50)
+  in_bounds :: "int \<Rightarrow> int \<Rightarrow> bool" (\<open>(_/ in'_bounds _)\<close> [50, 51] 50)
   where "i in_bounds k = (0 \<le> i \<and> i < k)"
 
 definition
@@ -306,11 +306,11 @@
 subsection "update"
 
 definition
-  gupd :: "oref  \<Rightarrow> obj \<Rightarrow> st \<Rightarrow> st" ("gupd'(_\<mapsto>_')" [10, 10] 1000)
+  gupd :: "oref  \<Rightarrow> obj \<Rightarrow> st \<Rightarrow> st" (\<open>gupd'(_\<mapsto>_')\<close> [10, 10] 1000)
   where "gupd r obj = case_st (\<lambda>g l. st (g(r\<mapsto>obj)) l)"
 
 definition
-  lupd :: "lname \<Rightarrow> val \<Rightarrow> st \<Rightarrow> st" ("lupd'(_\<mapsto>_')" [10, 10] 1000)
+  lupd :: "lname \<Rightarrow> val \<Rightarrow> st \<Rightarrow> st" (\<open>lupd'(_\<mapsto>_')\<close> [10, 10] 1000)
   where "lupd vn v = case_st (\<lambda>g l. st g (l(vn\<mapsto>v)))"
 
 definition