src/HOL/Eisbach/Eisbach_Tools.thy
changeset 63527 59eff6e56d81
parent 61853 fb7756087101
child 69593 3dda49e08b9d
--- a/src/HOL/Eisbach/Eisbach_Tools.thy	Wed Jul 20 11:11:07 2016 +0200
+++ b/src/HOL/Eisbach/Eisbach_Tools.thy	Wed Jul 20 11:44:11 2016 +0200
@@ -55,11 +55,11 @@
 \<close>
 
 method_setup catch = \<open>
-  Method_Closure.method_text -- Method_Closure.method_text >>
+  Method.text_closure -- Method.text_closure >>
     (fn (text, text') => fn ctxt => fn using => fn st =>
       let
-        val method = Method_Closure.method_evaluate text ctxt using;
-        val backup_results = Method_Closure.method_evaluate text' ctxt using st;
+        val method = Method.evaluate_runtime text ctxt using;
+        val backup_results = Method.evaluate_runtime text' ctxt using st;
       in
         (case try method st of
           SOME seq => try_map backup_results seq