src/HOL/Mirabelle/Actions/mirabelle_sledgehammer.ML
changeset 47532 8e1a120ed492
parent 47481 b5873d4ff1e2
child 47728 6ee015f6ea4b
equal deleted inserted replaced
47531:7fe7c7419489 47532:8e1a120ed492
   473                  is_built_in_const relevance_fudge relevance_override
   473                  is_built_in_const relevance_fudge relevance_override
   474                  chained_ths hyp_ts concl_t
   474                  chained_ths hyp_ts concl_t
   475         val problem =
   475         val problem =
   476           {state = st', goal = goal, subgoal = i,
   476           {state = st', goal = goal, subgoal = i,
   477            subgoal_count = Sledgehammer_Util.subgoal_count st,
   477            subgoal_count = Sledgehammer_Util.subgoal_count st,
   478            facts = facts |> map Sledgehammer_Provers.Untranslated_Fact,
   478            facts = facts |> map Sledgehammer_Provers.Untranslated_Fact}
   479            smt_filter = NONE}
       
   480       in prover params (K (K (K ""))) problem end)) ()
   479       in prover params (K (K (K ""))) problem end)) ()
   481       handle TimeLimit.TimeOut => failed ATP_Proof.TimedOut
   480       handle TimeLimit.TimeOut => failed ATP_Proof.TimedOut
   482            | Fail "inappropriate" => failed ATP_Proof.Inappropriate
   481            | Fail "inappropriate" => failed ATP_Proof.Inappropriate
   483     val time_prover = run_time |> Time.toMilliseconds
   482     val time_prover = run_time |> Time.toMilliseconds
   484     val msg = message (preplay ()) ^ message_tail
   483     val msg = message (preplay ()) ^ message_tail