| changeset 40786 | 0a54cfc9add3 |
| parent 37760 | 8380686be5cd |
| child 41413 | 64cd30d6b0b8 |
--- a/src/HOL/ex/While_Combinator_Example.thy Sat Nov 27 17:44:36 2010 -0800 +++ b/src/HOL/ex/While_Combinator_Example.thy Sun Nov 28 15:20:51 2010 +0100 @@ -28,7 +28,7 @@ apply (fastsimp 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 intro!: finite_Diff dest: monoD) +apply (blast dest: monoD) done