src/HOL/Bali/Term.thy
changeset 58887 38db8ddc0f57
parent 58310 91ea607a34d8
child 62042 6c6ccf573479
--- a/src/HOL/Bali/Term.thy	Sun Nov 02 17:58:35 2014 +0100
+++ b/src/HOL/Bali/Term.thy	Sun Nov 02 18:16:19 2014 +0100
@@ -2,7 +2,7 @@
     Author:     David von Oheimb
 *)
 
-header {* Java expressions and statements *}
+subsection {* Java expressions and statements *}
 
 theory Term imports Value Table begin
 
@@ -427,7 +427,7 @@
   apply auto
   done
 
-section {* Evaluation of unary operations *}
+subsubsection {* Evaluation of unary operations *}
 primrec eval_unop :: "unop \<Rightarrow> val \<Rightarrow> val"
 where
   "eval_unop UPlus v = Intg (the_Intg v)"
@@ -435,7 +435,7 @@
 | "eval_unop UBitNot v = Intg 42"                -- "FIXME: Not yet implemented"
 | "eval_unop UNot v = Bool (\<not> the_Bool v)"
 
-section {* Evaluation of binary operations *}
+subsubsection {* Evaluation of binary operations *}
 primrec eval_binop :: "binop \<Rightarrow> val \<Rightarrow> val \<Rightarrow> val"
 where
   "eval_binop Mul     v1 v2 = Intg ((the_Intg v1) * (the_Intg v2))"