src/HOL/Tools/Mirabelle/mirabelle_sledgehammer.ML
changeset 82364 5af097d05e99
parent 82233 3e972fc58373
equal deleted inserted replaced
82363:3a7fc54b50ca 82364:5af097d05e99
   214      change_data #> inc_sh_time_isa cpu_time)
   214      change_data #> inc_sh_time_isa cpu_time)
   215   end
   215   end
   216 
   216 
   217 end
   217 end
   218 
   218 
   219 val try0 = not o null o Try0.try0 (SOME (Time.fromSeconds 5)) []
   219 val try0 = not o null o Try0.try0 (SOME (Time.fromSeconds 5)) Try0.empty_facts
   220 
   220 
   221 fun make_action ({arguments, timeout, output_dir, ...} : Mirabelle.action_context) =
   221 fun make_action ({arguments, timeout, output_dir, ...} : Mirabelle.action_context) =
   222   let
   222   let
   223     (* Parse Mirabelle-specific parameters *)
   223     (* Parse Mirabelle-specific parameters *)
   224     val check_trivial =
   224     val check_trivial =