src/HOL/Eisbach/Eisbach_Tools.thy
changeset 61818 6de8e7ad95c3
parent 61268 abe08fb15a12
child 61853 fb7756087101
equal deleted inserted replaced
61817:6dde8fcd7f95 61818:6de8e7ad95c3
    53     | SOME NONE => Seq.empty
    53     | SOME NONE => Seq.empty
    54     | NONE => v);
    54     | NONE => v);
    55 \<close>
    55 \<close>
    56 
    56 
    57 method_setup catch = \<open>
    57 method_setup catch = \<open>
    58   Method_Closure.parse_method -- Method_Closure.parse_method >>
    58   Method_Closure.method_text -- Method_Closure.method_text >>
    59     (fn (text, text') => fn ctxt => fn using => fn st =>
    59     (fn (text, text') => fn ctxt => fn using => fn st =>
    60       let
    60       let
    61         val method = Method_Closure.method_evaluate text ctxt using;
    61         val method = Method_Closure.method_evaluate text ctxt using;
    62         val backup_results = Method_Closure.method_evaluate text' ctxt using st;
    62         val backup_results = Method_Closure.method_evaluate text' ctxt using st;
    63       in
    63       in