diff -r 6061ae1f90f2 -r 9bc16273c2d4 src/HOL/MicroJava/JVM/JVMExceptions.thy --- 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 \ cname \ p_count \ exception_entry \ bool"