src/HOL/Bali/WellForm.thy
changeset 44890 22f665a2e91c
parent 37956 ee939247b2fb
child 45605 a89b4bc311a5
--- a/src/HOL/Bali/WellForm.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Bali/WellForm.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -2788,7 +2788,7 @@
       proof -
         from im statM statT isT_statT wf not_Private_statM 
         have "is_static im = is_static statM"
-          by (fastsimp dest: wf_imethds_hiding_objmethdsD)
+          by (fastforce 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)