diff -r c86a47d4966e -r 2d9de77d5687 Quot/QuotMain.thy --- a/Quot/QuotMain.thy Wed Dec 09 05:59:49 2009 +0100 +++ b/Quot/QuotMain.thy Wed Dec 09 06:21:09 2009 +0100 @@ -1063,10 +1063,7 @@ fun simps thms = (mk_minimal_ss lthy) addsimps thms addSolver quotient_solver in EVERY' [simp_tac (simps thms1), - fun_map_tac lthy, - fun_map_tac lthy, - fun_map_tac lthy, - fun_map_tac lthy, + TRY o REPEAT_ALL_NEW (CHANGED o (fun_map_tac lthy)), lambda_prs_tac lthy, simp_tac (simps thms2), TRY o rtac refl]