src/HOL/IMP/Sec_Typing.thy
changeset 80914 d97fdabd9e2b
parent 69597 ff784d5a5bfb
--- a/src/HOL/IMP/Sec_Typing.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/IMP/Sec_Typing.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -7,7 +7,7 @@
 
 subsubsection "Syntax Directed Typing"
 
-inductive sec_type :: "nat \<Rightarrow> com \<Rightarrow> bool" ("(_/ \<turnstile> _)" [0,0] 50) where
+inductive sec_type :: "nat \<Rightarrow> com \<Rightarrow> bool" (\<open>(_/ \<turnstile> _)\<close> [0,0] 50) where
 Skip:
   "l \<turnstile> SKIP" |
 Assign:
@@ -183,7 +183,7 @@
 computation by an antimonotonicity rule. We introduce the standard system now
 and show the equivalence with our formulation.\<close>
 
-inductive sec_type' :: "nat \<Rightarrow> com \<Rightarrow> bool" ("(_/ \<turnstile>'' _)" [0,0] 50) where
+inductive sec_type' :: "nat \<Rightarrow> com \<Rightarrow> bool" (\<open>(_/ \<turnstile>'' _)\<close> [0,0] 50) where
 Skip':
   "l \<turnstile>' SKIP" |
 Assign':
@@ -217,7 +217,7 @@
 
 subsubsection "A Bottom-Up Typing System"
 
-inductive sec_type2 :: "com \<Rightarrow> level \<Rightarrow> bool" ("(\<turnstile> _ : _)" [0,0] 50) where
+inductive sec_type2 :: "com \<Rightarrow> level \<Rightarrow> bool" (\<open>(\<turnstile> _ : _)\<close> [0,0] 50) where
 Skip2:
   "\<turnstile> SKIP : l" |
 Assign2: