| changeset 61389 | 509d7ee638f8 |
| parent 61388 | 92e97b800d1e |
| child 61390 | a705f42b244d |
--- a/src/Cube/Example.thy Sat Oct 10 21:08:58 2015 +0200 +++ b/src/Cube/Example.thy Sat Oct 10 21:12:37 2015 +0200 @@ -19,7 +19,7 @@ method_setup strip_asms = \<open>Attrib.thms >> (fn thms => fn ctxt => METHOD (fn facts => - REPEAT (resolve_tac ctxt [@{thm strip_b}, @{thm strip_s}] 1 THEN + REPEAT (resolve_tac ctxt @{thms strip_b strip_s} 1 THEN DEPTH_SOLVE_1 (assume_tac ctxt 1 ORELSE resolve_tac ctxt (facts @ thms) 1))))\<close>