diff -r a273bdac0934 -r 8b5f00202e1a src/HOL/MicroJava/JVM/JVMExceptions.thy --- a/src/HOL/MicroJava/JVM/JVMExceptions.thy Wed Oct 07 19:45:00 2015 +0200 +++ b/src/HOL/MicroJava/JVM/JVMExceptions.thy Wed Oct 07 23:28:49 2015 +0200 @@ -3,7 +3,7 @@ Copyright 2001 Technische Universitaet Muenchen *) -section {* Exception handling in the JVM *} +section \Exception handling in the JVM\ theory JVMExceptions imports JVMInstructions begin @@ -41,15 +41,15 @@ | Some handler_pc \ (None, hp, ([xc], loc, C, sig, handler_pc)#frs)))" -text {* +text \ System exceptions are allocated in all heaps: -*} +\ -text {* +text \ Only program counters that are mentioned in the exception table can be returned by @{term match_exception_table}: -*} +\ lemma match_exception_table_in_et: "match_exception_table G C pc et = Some pc' \ \e \ set et. pc' = fst (snd (snd e))" by (induct et) (auto split: split_if_asm)