src/HOL/TPTP/atp_problem_import.ML
changeset 61310 9a50ea544fd3
parent 60543 ea2778854739
child 61569 947ce60a06e1
equal deleted inserted replaced
61309:a2548e708f03 61310:9a50ea544fd3
   114     fun print_szs_of_outcome falsify s =
   114     fun print_szs_of_outcome falsify s =
   115       "% SZS status " ^
   115       "% SZS status " ^
   116       (if s = "genuine" then
   116       (if s = "genuine" then
   117          if falsify then "CounterSatisfiable" else "Satisfiable"
   117          if falsify then "CounterSatisfiable" else "Satisfiable"
   118        else
   118        else
   119          "Unknown")
   119          "GaveUp")
   120       |> writeln
   120       |> writeln
   121     val (conjs, (defs, nondefs), ctxt) = read_tptp_file thy snd file_name
   121     val (conjs, (defs, nondefs), ctxt) = read_tptp_file thy snd file_name
   122     val params =
   122     val params =
   123       [("maxtime", string_of_int timeout),
   123       [("maxtime", string_of_int timeout),
   124        ("maxvars", "100000")]
   124        ("maxvars", "100000")]
   266 fun print_szs_of_success conjs success =
   266 fun print_szs_of_success conjs success =
   267   writeln ("% SZS status " ^
   267   writeln ("% SZS status " ^
   268     (if success then
   268     (if success then
   269        if null conjs then "Unsatisfiable" else "Theorem"
   269        if null conjs then "Unsatisfiable" else "Theorem"
   270      else
   270      else
   271        "Unknown"))
   271        "GaveUp"))
   272 
   272 
   273 fun sledgehammer_tptp_file thy timeout file_name =
   273 fun sledgehammer_tptp_file thy timeout file_name =
   274   let
   274   let
   275     val (conjs, assms, ctxt) = read_tptp_file thy (freeze_problem_consts thy o snd) file_name
   275     val (conjs, assms, ctxt) = read_tptp_file thy (freeze_problem_consts thy o snd) file_name
   276     val conj = make_conj ([], []) conjs
   276     val conj = make_conj ([], []) conjs