src/HOL/Tools/Mirabelle/mirabelle_try0.ML
author wenzelm
Sat, 15 May 2021 13:25:52 +0200
changeset 73694 60519a7bfc53
parent 73691 2f9877db82a1
child 73847 58f6b41efe88
permissions -rw-r--r--
clarified signature; supporess empty results;

(*  Title:      HOL/Mirabelle/Tools/mirabelle_try0.ML
    Author:     Jasmin Blanchette, TU Munich
    Author:     Makarius

Mirabelle action: "try0".
*)

structure Mirabelle_Try0 : sig end =
struct

val _ =
  Theory.setup (Mirabelle.command_action \<^binding>\<open>try0\<close>
    (fn {timeout, ...} => fn {pre, ...} =>
      if Timeout.apply (Time.scale 10.0 timeout) (Try0.try0 (SOME timeout) ([], [], [], [])) pre
      then "succeeded" else ""));

end