changeset 19931 | fb32b43e7f80 |
parent 17453 | eccff680177d |
child 19943 | 26b37721b357 |
--- a/src/Cube/Example.thy Tue Jun 20 14:51:59 2006 +0200 +++ b/src/Cube/Example.thy Tue Jun 20 15:53:44 2006 +0200 @@ -16,7 +16,7 @@ method_setup depth_solve = {* Method.thms_args (fn thms => Method.METHOD (fn facts => - (DEPTH_SOLVE (HEADGOAL (ares_tac (facts @ thms)))))) + (DEPTH_SOLVE (HEADGOAL (ares_tac (PolyML.print (facts @ thms))))))) *} "" method_setup depth_solve1 = {*