src/HOL/MicroJava/JVM/JVMExceptions.thy
changeset 16417 9bc16273c2d4
parent 13674 f4c64597fb02
child 35102 cc7a0b9f938c
--- a/src/HOL/MicroJava/JVM/JVMExceptions.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/MicroJava/JVM/JVMExceptions.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* \isaheader{Exception handling in the JVM} *}
 
-theory JVMExceptions = JVMInstructions:
+theory JVMExceptions imports JVMInstructions begin
 
 constdefs
   match_exception_entry :: "jvm_prog \<Rightarrow> cname \<Rightarrow> p_count \<Rightarrow> exception_entry \<Rightarrow> bool"