in wellformed programs, exceptions are classes
authorkleing
Sat, 09 Mar 2002 20:39:19 +0100
changeset 13051 8efb5d92cf55
parent 13050 04deb0c8dcbe
child 13052 3bf41c474a88
in wellformed programs, exceptions are classes
src/HOL/MicroJava/J/WellForm.thy
--- a/src/HOL/MicroJava/J/WellForm.thy	Fri Mar 08 20:39:39 2002 +0100
+++ b/src/HOL/MicroJava/J/WellForm.thy	Sat Mar 09 20:39:19 2002 +0100
@@ -70,6 +70,15 @@
 apply (simp (no_asm_simp))
 done
 
+lemma is_class_xcpt [simp]: "wf_prog wf_mb G \<Longrightarrow> is_class G (Xcpt x)"
+  apply (simp add: wf_prog_def wf_syscls_def)
+  apply (simp add: is_class_def class_def)
+  apply clarify
+  apply (erule_tac x = x in allE)
+  apply clarify
+  apply (auto intro!: map_of_SomeI)
+  done
+
 lemma subcls1_wfD: "[|G\<turnstile>C\<prec>C1D; wf_prog wf_mb G|] ==> D \<noteq> C \<and> \<not>(D,C)\<in>(subcls1 G)^+"
 apply( frule r_into_trancl)
 apply( drule subcls1D)