src/HOL/IMP/Sec_Typing.thy
changeset 68776 403dd13cf6e9
parent 67406 23307fd33906
child 69597 ff784d5a5bfb
--- a/src/HOL/IMP/Sec_Typing.thy	Fri Aug 17 11:26:35 2018 +0000
+++ b/src/HOL/IMP/Sec_Typing.thy	Mon Aug 20 20:54:26 2018 +0200
@@ -1,9 +1,11 @@
 (* Author: Tobias Nipkow *)
 
+subsection "Security Typing of Commands"
+
 theory Sec_Typing imports Sec_Type_Expr
 begin
 
-subsection "Syntax Directed Typing"
+subsubsection "Syntax Directed Typing"
 
 inductive sec_type :: "nat \<Rightarrow> com \<Rightarrow> bool" ("(_/ \<turnstile> _)" [0,0] 50) where
 Skip:
@@ -174,7 +176,7 @@
 qed
 
 
-subsection "The Standard Typing System"
+subsubsection "The Standard Typing System"
 
 text\<open>The predicate @{prop"l \<turnstile> c"} is nicely intuitive and executable. The
 standard formulation, however, is slightly different, replacing the maximum
@@ -213,7 +215,7 @@
 apply (metis max.absorb2 While)
 by (metis anti_mono)
 
-subsection "A Bottom-Up Typing System"
+subsubsection "A Bottom-Up Typing System"
 
 inductive sec_type2 :: "com \<Rightarrow> level \<Rightarrow> bool" ("(\<turnstile> _ : _)" [0,0] 50) where
 Skip2: