src/HOL/IMP/Sec_TypingT.thy
changeset 68776 403dd13cf6e9
parent 67406 23307fd33906
child 69597 ff784d5a5bfb
--- a/src/HOL/IMP/Sec_TypingT.thy	Fri Aug 17 11:26:35 2018 +0000
+++ b/src/HOL/IMP/Sec_TypingT.thy	Mon Aug 20 20:54:26 2018 +0200
@@ -1,7 +1,9 @@
+subsection "Termination-Sensitive Systems"
+
 theory Sec_TypingT imports Sec_Type_Expr
 begin
 
-subsection "A Termination-Sensitive Syntax Directed System"
+subsubsection "A Syntax Directed System"
 
 inductive sec_type :: "nat \<Rightarrow> com \<Rightarrow> bool" ("(_/ \<turnstile> _)" [0,0] 50) where
 Skip:
@@ -163,7 +165,7 @@
     by (metis \<open>s' = t' (\<le> l)\<close>)
 qed
 
-subsection "The Standard Termination-Sensitive System"
+subsubsection "The Standard System"
 
 text\<open>The predicate @{prop"l \<turnstile> c"} is nicely intuitive and executable. The
 standard formulation, however, is slightly different, replacing the maximum