src/HOL/Bali/AxSound.thy
changeset 58887 38db8ddc0f57
parent 55524 f41ef840f09d
child 58963 26bf09b95dda
--- a/src/HOL/Bali/AxSound.thy	Sun Nov 02 17:58:35 2014 +0100
+++ b/src/HOL/Bali/AxSound.thy	Sun Nov 02 18:16:19 2014 +0100
@@ -1,13 +1,13 @@
 (*  Title:      HOL/Bali/AxSound.thy
     Author:     David von Oheimb and Norbert Schirmer
 *)
-header {* Soundness proof for Axiomatic semantics of Java expressions and 
+subsection {* Soundness proof for Axiomatic semantics of Java expressions and 
           statements
        *}
 
 theory AxSound imports AxSem begin
 
-section "validity"
+subsubsection "validity"
 
 definition
   triple_valid2 :: "prog \<Rightarrow> nat \<Rightarrow> 'a triple \<Rightarrow> bool"  ("_\<Turnstile>_\<Colon>_"[61,0, 58] 57)
@@ -100,7 +100,7 @@
 oops
 
 
-section "soundness"
+subsubsection "soundness"
 
 lemma Methd_sound: 
   assumes recursive: "G,A\<union>  {{P} Methd-\<succ> {Q} | ms}|\<Turnstile>\<Colon>{{P} body G-\<succ> {Q} | ms}"