src/HOL/TPTP/TPTP_Parser/tptp_reconstruct.ML
changeset 62519 a564458f94db
parent 62243 dd22d2423047
child 62552 53603d1aad5f
equal deleted inserted replaced
62518:b8efcc9edd7b 62519:a564458f94db
  1058         fun rest memo' ctxt' = skel_to_naive_tactic_dbg prover_tac ctxt' prob_name (tl skel) memo'
  1058         fun rest memo' ctxt' = skel_to_naive_tactic_dbg prover_tac ctxt' prob_name (tl skel) memo'
  1059         (*reconstruct the inference. also set timeout in case
  1059         (*reconstruct the inference. also set timeout in case
  1060           tactic takes too long*)
  1060           tactic takes too long*)
  1061         val try_make_step =
  1061         val try_make_step =
  1062           (*FIXME const timeout*)
  1062           (*FIXME const timeout*)
  1063           (* TimeLimit.timeLimit (Time.fromSeconds 5) *)
  1063           (* Timeout.apply (Time.fromSeconds 5) *)
  1064           (fn ctxt' =>
  1064           (fn ctxt' =>
  1065              let
  1065              let
  1066                fun thm ctxt'' = prover_tac ctxt'' prob_name (hd skel |> stock_to_string)
  1066                fun thm ctxt'' = prover_tac ctxt'' prob_name (hd skel |> stock_to_string)
  1067                val reconstructed_inference = thm ctxt'
  1067                val reconstructed_inference = thm ctxt'
  1068                fun rec_inf_tac st = HEADGOAL (resolve_tac ctxt' [thm ctxt']) st
  1068                fun rec_inf_tac st = HEADGOAL (resolve_tac ctxt' [thm ctxt']) st