src/HOL/MicroJava/BV/Altern.thy
changeset 33954 1bc3b688548c
parent 26450 158b924b5153
child 35416 d8d7d1b785af
--- a/src/HOL/MicroJava/BV/Altern.thy	Wed Dec 02 12:04:07 2009 +0100
+++ b/src/HOL/MicroJava/BV/Altern.thy	Tue Nov 24 14:37:23 2009 +0100
@@ -1,15 +1,12 @@
 (*  Title:      HOL/MicroJava/BV/Altern.thy
-    ID:         $Id$
     Author:     Martin Strecker
 *)
 
-
-(* Alternative definition of well-typing of bytecode, 
-   used in compiler type correctness proof *)
+header {* Alternative definition of well-typing of bytecode,  used in compiler type correctness proof *}
 
-
-theory Altern imports BVSpec begin
-
+theory Altern
+imports BVSpec
+begin
 
 constdefs
   check_type :: "jvm_prog \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> JVMType.state \<Rightarrow> bool"