src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 41315 7f6baec2b27a
parent 41313 a96ac4d180b7
child 41318 adcb92c0513b
equal deleted inserted replaced
41314:2dc1dfc1bc69 41315:7f6baec2b27a
   358         Path.append (Path.explode dest_dir) problem_file_name
   358         Path.append (Path.explode dest_dir) problem_file_name
   359       else
   359       else
   360         error ("No such directory: " ^ quote dest_dir ^ ".")
   360         error ("No such directory: " ^ quote dest_dir ^ ".")
   361     val measure_run_time = verbose orelse Config.get ctxt measure_run_time
   361     val measure_run_time = verbose orelse Config.get ctxt measure_run_time
   362     val command = Path.explode (getenv (fst exec) ^ "/" ^ snd exec)
   362     val command = Path.explode (getenv (fst exec) ^ "/" ^ snd exec)
   363 val command = Path.explode ("/Users/blanchet/misc/E-weights/PROVER/" ^ snd exec) (*###*)
       
   364     fun split_time s =
   363     fun split_time s =
   365       let
   364       let
   366         val split = String.tokens (fn c => str c = "\n");
   365         val split = String.tokens (fn c => str c = "\n");
   367         val (output, t) = s |> split |> split_last |> apfst cat_lines;
   366         val (output, t) = s |> split |> split_last |> apfst cat_lines;
   368         fun as_num f = f >> (fst o read_int);
   367         fun as_num f = f >> (fst o read_int);