src/Cube/Example.thy
changeset 19943 26b37721b357
parent 19931 fb32b43e7f80
child 30510 4120fc59dd85
equal deleted inserted replaced
19942:dc92e3aebc71 19943:26b37721b357
    14   J. Functional Programming.
    14   J. Functional Programming.
    15 *}
    15 *}
    16 
    16 
    17 method_setup depth_solve = {*
    17 method_setup depth_solve = {*
    18   Method.thms_args (fn thms => Method.METHOD (fn facts =>
    18   Method.thms_args (fn thms => Method.METHOD (fn facts =>
    19   (DEPTH_SOLVE (HEADGOAL (ares_tac (PolyML.print (facts @ thms)))))))
    19   (DEPTH_SOLVE (HEADGOAL (ares_tac (facts @ thms))))))
    20 *} ""
    20 *} ""
    21 
    21 
    22 method_setup depth_solve1 = {*
    22 method_setup depth_solve1 = {*
    23   Method.thms_args (fn thms => Method.METHOD (fn facts =>
    23   Method.thms_args (fn thms => Method.METHOD (fn facts =>
    24   (DEPTH_SOLVE_1 (HEADGOAL (ares_tac (facts @ thms))))))
    24   (DEPTH_SOLVE_1 (HEADGOAL (ares_tac (facts @ thms))))))