src/HOL/Bali/WellForm.thy
changeset 13601 fd3e3d6b37b2
parent 12963 73fb6a200e36
child 13688 a0b16d42d489
--- a/src/HOL/Bali/WellForm.thy	Mon Sep 30 16:12:16 2002 +0200
+++ b/src/HOL/Bali/WellForm.thy	Mon Sep 30 16:14:02 2002 +0200
@@ -1420,10 +1420,10 @@
   show "?Class C \<Longrightarrow> ?Method C \<Longrightarrow> ?MemberOf C"
   proof (induct rule: ws_class_induct')  
     case Object
-    with wf have declC: "declclass m = Object"
-      by (blast intro: declclass_methd_Object)
-    with Object wf have "G\<turnstile>Methd sig m declared_in Object"
-      by (auto dest: methd_declaredD simp del: methd_Object)
+    with wf have declC: "Object = declclass m"
+      by (simp add: declclass_methd_Object)
+    from Object wf have "G\<turnstile>Methd sig m declared_in Object"
+      by (auto intro: methd_declaredD simp add: declC)
     with declC 
     show "?MemberOf Object"
       by (auto intro!: members.Immediate
@@ -2794,7 +2794,7 @@
       proof -
 	from im statM statT isT_statT wf not_Private_statM 
 	have "is_static im = is_static statM"
-	  by (auto dest: wf_imethds_hiding_objmethdsD)
+	  by (fastsimp dest: wf_imethds_hiding_objmethdsD)
 	with wf isT_statT statT im 
 	have "\<not> is_static statM"
 	  by (auto dest: wf_prog_idecl imethds_wf_mhead)