src/HOL/TLA/Init.thy
changeset 80914 d97fdabd9e2b
parent 62146 324bc1ffba12
--- a/src/HOL/TLA/Init.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/TLA/Init.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -25,8 +25,8 @@
   where Init_def: "Initial F sigma = F (first_world sigma)"
 
 syntax
-  "_TEMP"    :: "lift \<Rightarrow> 'a"                          ("(TEMP _)")
-  "_Init"    :: "lift \<Rightarrow> lift"                        ("(Init _)"[40] 50)
+  "_TEMP"    :: "lift \<Rightarrow> 'a"                          (\<open>(TEMP _)\<close>)
+  "_Init"    :: "lift \<Rightarrow> lift"                        (\<open>(Init _)\<close>[40] 50)
 translations
   "TEMP F"   => "(F::behavior \<Rightarrow> _)"
   "_Init"    == "CONST Initial"