src/HOL/Bali/Decl.thy
changeset 58887 38db8ddc0f57
parent 58310 91ea607a34d8
child 61989 ba8c284d4725
--- a/src/HOL/Bali/Decl.thy	Sun Nov 02 17:58:35 2014 +0100
+++ b/src/HOL/Bali/Decl.thy	Sun Nov 02 18:16:19 2014 +0100
@@ -1,7 +1,7 @@
 (*  Title:      HOL/Bali/Decl.thy
     Author:     David von Oheimb and Norbert Schirmer
 *)
-header {* Field, method, interface, and class declarations, whole Java programs
+subsection {* Field, method, interface, and class declarations, whole Java programs
 *}
 
 theory Decl
@@ -367,7 +367,7 @@
 by (simp add: cbody_def)
 
 
-section "standard classes"
+subsubsection "standard classes"
 
 consts
   Object_mdecls  ::  "mdecl list" --{* methods of Object *}
@@ -399,7 +399,7 @@
                 SXcptC NegArrSize , SXcptC IndOutBound, SXcptC ArrStore]"
 
 
-section "programs"
+subsubsection "programs"
 
 record prog =
         ifaces ::"idecl list"
@@ -426,7 +426,7 @@
   where "is_class G C == class G C \<noteq> None"
 
 
-section "is type"
+subsubsection "is type"
 
 primrec is_type :: "prog \<Rightarrow> ty \<Rightarrow> bool"
   and isrtype :: "prog \<Rightarrow> ref_ty \<Rightarrow> bool"
@@ -445,7 +445,7 @@
 by auto
 
 
-section "subinterface and subclass relation, in anticipation of TypeRel.thy"
+subsubsection "subinterface and subclass relation, in anticipation of TypeRel.thy"
 
 definition
   subint1  :: "prog \<Rightarrow> (qtname \<times> qtname) set" --{* direct subinterface *}
@@ -516,7 +516,7 @@
 apply (auto intro: no_subcls1_Object)
 done
 
-section "well-structured programs"
+subsubsection "well-structured programs"
 
 definition
   ws_idecl :: "prog \<Rightarrow> qtname \<Rightarrow> qtname list \<Rightarrow> bool"
@@ -562,7 +562,7 @@
 done
 
 
-section "well-foundedness"
+subsubsection "well-foundedness"
 
 lemma finite_is_iface: "finite {I. is_iface G I}"
 apply (fold dom_def)
@@ -765,7 +765,7 @@
   qed
 qed
 
-section "general recursion operators for the interface and class hiearchies"
+subsubsection "general recursion operators for the interface and class hiearchies"
 
 function iface_rec  :: "prog \<Rightarrow> qtname \<Rightarrow> (qtname \<Rightarrow> iface \<Rightarrow> 'a set \<Rightarrow> 'a) \<Rightarrow> 'a"
 where