diff -r 8a6cac7c7247 -r 38db8ddc0f57 src/HOL/Bali/TypeRel.thy --- a/src/HOL/Bali/TypeRel.thy Sun Nov 02 17:58:35 2014 +0100 +++ b/src/HOL/Bali/TypeRel.thy Sun Nov 02 18:16:19 2014 +0100 @@ -1,7 +1,7 @@ (* Title: HOL/Bali/TypeRel.thy Author: David von Oheimb *) -header {* The relations between Java types *} +subsection {* The relations between Java types *} theory TypeRel imports Decl begin @@ -55,7 +55,7 @@ implmt1_syntax ("_\_\1_" [71,71,71] 70) -section "subclass and subinterface relations" +subsubsection "subclass and subinterface relations" (* direct subinterface in Decl.thy, cf. 9.1.3 *) (* direct subclass in Decl.thy, cf. 8.1.3 *) @@ -327,7 +327,7 @@ qed qed -section "implementation relation" +subsubsection "implementation relation" lemma implmt1D: "G\C\1I \ C\Object \ (\c\class G C: I\set (superIfs c))" apply (unfold implmt1_def) @@ -366,7 +366,7 @@ done -section "widening relation" +subsubsection "widening relation" inductive --{*widening, viz. method invocation conversion, cf. 5.3 @@ -583,7 +583,7 @@ done -section "narrowing relation" +subsubsection "narrowing relation" (* all properties of narrowing and casting conversions we actually need *) (* these can easily be proven from the definitions below *) @@ -643,7 +643,7 @@ lemma narrow_Boolean2: "G\S\PrimT Boolean \ S=PrimT Boolean" by (ind_cases "G\S\PrimT Boolean") -section "casting relation" +subsubsection "casting relation" inductive --{* casting conversion, cf. 5.5 *} cast :: "prog \ ty \ ty \ bool" ("_\_\? _" [71,71,71] 70)