diff -r 50b60f501b05 -r 14095f771781 src/Cube/Example.thy --- a/src/Cube/Example.thy Tue Feb 10 14:48:26 2015 +0100 +++ b/src/Cube/Example.thy Tue Feb 10 16:46:21 2015 +0100 @@ -10,17 +10,17 @@ J. Functional Programming.\ method_setup depth_solve = - \Attrib.thms >> (fn thms => K (METHOD (fn facts => - (DEPTH_SOLVE (HEADGOAL (ares_tac (facts @ thms)))))))\ + \Attrib.thms >> (fn thms => fn ctxt => METHOD (fn facts => + (DEPTH_SOLVE (HEADGOAL (assume_tac ctxt ORELSE' resolve_tac ctxt (facts @ thms))))))\ method_setup depth_solve1 = - \Attrib.thms >> (fn thms => K (METHOD (fn facts => - (DEPTH_SOLVE_1 (HEADGOAL (ares_tac (facts @ thms)))))))\ + \Attrib.thms >> (fn thms => fn ctxt => METHOD (fn facts => + (DEPTH_SOLVE_1 (HEADGOAL (assume_tac ctxt ORELSE' resolve_tac ctxt (facts @ thms))))))\ method_setup strip_asms = \Attrib.thms >> (fn thms => fn ctxt => METHOD (fn facts => REPEAT (resolve_tac ctxt [@{thm strip_b}, @{thm strip_s}] 1 THEN - DEPTH_SOLVE_1 (ares_tac (facts @ thms) 1))))\ + DEPTH_SOLVE_1 (assume_tac ctxt 1 ORELSE resolve_tac ctxt (facts @ thms) 1))))\ subsection \Simple types\