src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML
changeset 62601 a937889f0086
parent 61312 6d779a71086d
child 62925 f1bdf10f95d8
equal deleted inserted replaced
62600:614aefb0e6cc 62601:a937889f0086
   313 
   313 
   314     val thy = Proof.theory_of state
   314     val thy = Proof.theory_of state
   315     val ctxt = Proof.context_of state
   315     val ctxt = Proof.context_of state
   316 
   316 
   317     val override_params = override_params |> map (normalize_raw_param ctxt)
   317     val override_params = override_params |> map (normalize_raw_param ctxt)
   318     val _ = Isabelle_System.mkdir (Path.explode (getenv "ISABELLE_TMP"))
       
   319   in
   318   in
   320     if subcommand = runN then
   319     if subcommand = runN then
   321       let val i = the_default 1 opt_i in
   320       let val i = the_default 1 opt_i in
   322         ignore (run_sledgehammer
   321         ignore (run_sledgehammer
   323           (get_params Normal thy override_params) Normal writeln_result i fact_override state)
   322           (get_params Normal thy override_params) Normal writeln_result i fact_override state)