src/HOL/Tools/Mirabelle/mirabelle_arith.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_arith.ML
    Author:     Jasmin Blanchette and Sascha Boehme, TU Munich
    Author:     Makarius

Mirabelle action: "arith".
*)

structure Mirabelle_Arith: sig end =
struct

val _ =
  Theory.setup (Mirabelle.command_action \<^binding>\<open>arith\<close>
    (fn {timeout, ...} => fn {pre, ...} =>
      if Mirabelle.can_apply timeout Arith_Data.arith_tac pre
      then "succeeded" else ""));

end