src/HOL/UNITY/WFair.thy
changeset 19769 c40ce2de2020
parent 16417 9bc16273c2d4
child 23767 7272a839ccd9
--- a/src/HOL/UNITY/WFair.thy	Sun Jun 04 10:52:47 2006 +0200
+++ b/src/HOL/UNITY/WFair.thy	Mon Jun 05 14:22:58 2006 +0200
@@ -492,7 +492,7 @@
       ==> F \<in> A leadsTo ((A \<inter> (f-`(atLeast l))) \<union> B)"
 apply (rule_tac f = f and f1 = "%k. l - k" 
        in wf_less_than [THEN wf_inv_image, THEN leadsTo_wf_induct])
-apply (simp (no_asm) add: inv_image_def Image_singleton)
+apply (simp (no_asm) add:Image_singleton)
 apply clarify
 apply (case_tac "m<l")
  apply (blast intro: leadsTo_weaken_R diff_less_mono2)