src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML
changeset 58075 95bab16eac45
parent 58028 e4250d370657
child 58089 20e76da3a0ef
equal deleted inserted replaced
58074:87a8cc594bf6 58075:95bab16eac45
   314 
   314 
   315 (* Sledgehammer the given subgoal *)
   315 (* Sledgehammer the given subgoal *)
   316 
   316 
   317 val default_learn_prover_timeout = 2.0
   317 val default_learn_prover_timeout = 2.0
   318 
   318 
   319 fun hammer_away override_params subcommand opt_i fact_override state =
   319 fun hammer_away override_params subcommand opt_i fact_override state0 =
   320   let
   320   let
       
   321     val state = state0
       
   322       |> Proof.map_contexts (Try0.silence_methods false #> Config.put SMT_Config.verbose false)
   321     val thy = Proof.theory_of state
   323     val thy = Proof.theory_of state
   322     val ctxt = Proof.context_of state
   324     val ctxt = Proof.context_of state
   323 
   325 
   324     val override_params = override_params |> map (normalize_raw_param ctxt)
   326     val override_params = override_params |> map (normalize_raw_param ctxt)
   325     val _ = Isabelle_System.mkdir (Path.explode (getenv "ISABELLE_TMP"))
   327     val _ = Isabelle_System.mkdir (Path.explode (getenv "ISABELLE_TMP"))