src/HOL/Tools/try0.ML
changeset 79742 2e4518e8a36b
parent 78239 4fe65149f3fd
child 79743 3648e9c88d0c
equal deleted inserted replaced
79741:513829904beb 79742:2e4518e8a36b
   107   Config.put Metis_Tactic.verbose debug
   107   Config.put Metis_Tactic.verbose debug
   108   #> not debug ? (fn ctxt =>
   108   #> not debug ? (fn ctxt =>
   109       ctxt
   109       ctxt
   110       |> Simplifier_Trace.disable
   110       |> Simplifier_Trace.disable
   111       |> Context_Position.set_visible false
   111       |> Context_Position.set_visible false
   112       |> Config.put Unify.trace_bound (Config.get ctxt Unify.search_bound)
   112       |> Config.put Unify.unify_trace_bound (Config.get ctxt Unify.search_bound)
   113       |> Config.put Argo_Tactic.trace "none"
   113       |> Config.put Argo_Tactic.trace "none"
   114       |> Proof_Context.background_theory (fn thy =>
   114       |> Proof_Context.background_theory (fn thy =>
   115           thy
   115           thy
   116           |> Context_Position.set_visible_global false
   116           |> Context_Position.set_visible_global false
   117           |> Config.put_global Unify.trace_bound (Config.get_global thy Unify.search_bound)));
   117           |> Config.put_global Unify.unify_trace_bound (Config.get_global thy Unify.search_bound)));
   118 
   118 
   119 fun generic_try0 mode timeout_opt quad st =
   119 fun generic_try0 mode timeout_opt quad st =
   120   let
   120   let
   121     val st = Proof.map_contexts (silence_methods false) st;
   121     val st = Proof.map_contexts (silence_methods false) st;
   122     fun trd (_, _, t) = t;
   122     fun trd (_, _, t) = t;