src/HOL/Eisbach/Eisbach_Tools.thy
changeset 61818 6de8e7ad95c3
parent 61268 abe08fb15a12
child 61853 fb7756087101
--- a/src/HOL/Eisbach/Eisbach_Tools.thy	Wed Dec 09 18:59:39 2015 +0100
+++ b/src/HOL/Eisbach/Eisbach_Tools.thy	Wed Dec 09 20:21:13 2015 +0100
@@ -55,7 +55,7 @@
 \<close>
 
 method_setup catch = \<open>
-  Method_Closure.parse_method -- Method_Closure.parse_method >>
+  Method_Closure.method_text -- Method_Closure.method_text >>
     (fn (text, text') => fn ctxt => fn using => fn st =>
       let
         val method = Method_Closure.method_evaluate text ctxt using;