src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 52196 2281f33e8da6
parent 52150 41c885784e04
child 52555 6811291d1869
equal deleted inserted replaced
52195:056ec8201667 52196:2281f33e8da6
   684     val thy = Proof.theory_of state
   684     val thy = Proof.theory_of state
   685     val ctxt = Proof.context_of state
   685     val ctxt = Proof.context_of state
   686     val atp_mode =
   686     val atp_mode =
   687       if Config.get ctxt completish then Sledgehammer_Completish
   687       if Config.get ctxt completish then Sledgehammer_Completish
   688       else Sledgehammer
   688       else Sledgehammer
   689     val ((_, hyp_ts, concl_t), ctxt') = strip_subgoal goal subgoal ctxt
   689     val (_, hyp_ts, concl_t) = strip_subgoal goal subgoal ctxt
   690     val (dest_dir, problem_prefix) =
   690     val (dest_dir, problem_prefix) =
   691       if overlord then overlord_file_location_of_prover name
   691       if overlord then overlord_file_location_of_prover name
   692       else (Config.get ctxt dest_dir, Config.get ctxt problem_prefix)
   692       else (Config.get ctxt dest_dir, Config.get ctxt problem_prefix)
   693     val problem_file_name =
   693     val problem_file_name =
   694       Path.basic (problem_prefix ^ (if overlord then "" else serial_string ()) ^
   694       Path.basic (problem_prefix ^ (if overlord then "" else serial_string ()) ^