diff -r 340df9f3491f -r 22f665a2e91c src/HOL/TPTP/CASC_Setup.thy --- a/src/HOL/TPTP/CASC_Setup.thy Sun Sep 11 22:56:05 2011 +0200 +++ b/src/HOL/TPTP/CASC_Setup.thy Mon Sep 12 07:55:43 2011 +0200 @@ -141,7 +141,7 @@ ORELSE SOLVE_TIMEOUT (max_secs div 10) "force" (ALLGOALS (force_tac ctxt)) ORELSE - SOLVE_TIMEOUT max_secs "fastsimp" (ALLGOALS (fast_simp_tac ctxt)) + SOLVE_TIMEOUT max_secs "fastforce" (ALLGOALS (fast_force_tac ctxt)) *} method_setup isabellep = {*