src/HOL/Eisbach/Eisbach_Tools.thy
changeset 60553 86fc6652c4df
parent 60285 b4f1a0a701ae
child 61268 abe08fb15a12
--- a/src/HOL/Eisbach/Eisbach_Tools.thy	Mon Jun 22 17:44:43 2015 +0200
+++ b/src/HOL/Eisbach/Eisbach_Tools.thy	Mon Jun 22 18:55:47 2015 +0200
@@ -14,7 +14,8 @@
 fun trace_method parser print =
   Scan.lift (Args.mode "dummy") -- parser >>
     (fn (dummy, x) => fn ctxt => SIMPLE_METHOD (fn st =>
-      (if dummy orelse not (Method_Closure.is_dummy st) then tracing (print ctxt x) else ();
+      (if dummy orelse not (Method.detect_closure_state st)
+       then tracing (print ctxt x) else ();
        all_tac st)));
 
 fun setup_trace_method binding parser print =