| changeset 44890 | 22f665a2e91c | 
| parent 41959 | b460124855b8 | 
| child 58889 | 5b7a9633cfa8 | 
--- a/src/HOL/ex/While_Combinator_Example.thy Sun Sep 11 22:56:05 2011 +0200 +++ b/src/HOL/ex/While_Combinator_Example.thy Mon Sep 12 07:55:43 2011 +0200 @@ -25,7 +25,7 @@ apply assumption apply clarsimp apply (blast dest: monoD) - apply (fastsimp intro!: lfp_lowerbound) + apply (fastforce intro!: lfp_lowerbound) apply (blast intro: wf_finite_psubset Int_lower2 [THEN [2] wf_subset]) apply (clarsimp simp add: finite_psubset_def order_less_le) apply (blast dest: monoD)