changeset 44890 | 22f665a2e91c |
parent 44106 | 0e018cbcc0de |
child 46911 | 6d2a2f0e904e |
--- a/src/HOL/UNITY/Transformers.thy Sun Sep 11 22:56:05 2011 +0200 +++ b/src/HOL/UNITY/Transformers.thy Mon Sep 12 07:55:43 2011 +0200 @@ -440,7 +440,7 @@ apply (rule subsetI) apply (erule wens_set.induct) txt{*Basis*} - apply (fastsimp simp add: wens_single_finite_def) + apply (fastforce simp add: wens_single_finite_def) txt{*Wens inductive step*} apply (case_tac "acta = Id", simp) apply (simp add: wens_single_eq)