src/HOL/TPTP/atp_problem_import.ML
changeset 47811 1e8eb643540d
parent 47794 4ad62c5f9f88
child 47812 bb477988edb4
equal deleted inserted replaced
47810:9579464d00f9 47811:1e8eb643540d
   138   Sledgehammer_Tactics.sledgehammer_as_oracle_tac ctxt
   138   Sledgehammer_Tactics.sledgehammer_as_oracle_tac ctxt
   139       ([("debug", if debug then "true" else "false"),
   139       ([("debug", if debug then "true" else "false"),
   140         ("overlord", if overlord then "true" else "false"),
   140         ("overlord", if overlord then "true" else "false"),
   141         ("provers", prover),
   141         ("provers", prover),
   142         ("timeout", string_of_int timeout)] @ override_params)
   142         ("timeout", string_of_int timeout)] @ override_params)
   143       {add = [], del = [], only = true}
   143       {add = [(Facts.named (Thm.derivation_name ext), [])],
       
   144        del = [], only = true}
   144 
   145 
   145 fun sledgehammer_tac ctxt timeout i =
   146 fun sledgehammer_tac ctxt timeout i =
   146   let
   147   let
   147     fun slice overload_params fraq prover =
   148     fun slice overload_params fraq prover =
   148       SOLVE_TIMEOUT (timeout div fraq) prover
   149       SOLVE_TIMEOUT (timeout div fraq) prover
   205   let
   206   let
   206     val (conjs, assms, ctxt) =
   207     val (conjs, assms, ctxt) =
   207       read_tptp_file thy (freeze_problem_consts thy) file_name
   208       read_tptp_file thy (freeze_problem_consts thy) file_name
   208     val conj = make_conj assms conjs
   209     val conj = make_conj assms conjs
   209   in
   210   in
   210     (can_tac ctxt (sledgehammer_tac ctxt (timeout div 2) 1) conj orelse
   211     (can_tac ctxt (auto_etc_tac ctxt (timeout div 2) 1) conj orelse
   211      can_tac ctxt (auto_etc_tac ctxt (timeout div 2) 1) conj orelse
   212      can_tac ctxt (sledgehammer_tac ctxt (timeout div 2) 1) conj orelse
   212      can_tac ctxt (atp_tac ctxt [] timeout ATP_Systems.satallaxN 1) conj)
   213      can_tac ctxt (atp_tac ctxt [] timeout ATP_Systems.satallaxN 1) conj)
   213     |> print_szs_from_success conjs
   214     |> print_szs_from_success conjs
   214   end
   215   end
   215 
   216 
   216 (** Translator between TPTP(-like) file formats **)
   217 (** Translator between TPTP(-like) file formats **)