more about match_exception_table
authorkleing
Sun, 24 Mar 2002 14:05:53 +0100
changeset 13065 d6585b32412b
parent 13064 1f54a5fecaa6
child 13066 b57d926d1de2
more about match_exception_table
src/HOL/MicroJava/JVM/JVMExceptions.thy
--- a/src/HOL/MicroJava/JVM/JVMExceptions.thy	Thu Mar 21 16:40:18 2002 +0100
+++ b/src/HOL/MicroJava/JVM/JVMExceptions.thy	Sun Mar 24 14:05:53 2002 +0100
@@ -87,4 +87,14 @@
   apply (auto simp add: blank_def)
   done
 
+
+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' \<Longrightarrow> \<exists>e \<in> set et. pc' = fst (snd (snd e))"
+  by (induct et) (auto split: split_if_asm)
+
+
 end