src/HOL/Tools/Mirabelle/mirabelle_arith.ML
author wenzelm
Fri, 14 May 2021 21:32:11 +0200
changeset 73691 2f9877db82a1
parent 62519 src/HOL/Mirabelle/Tools/mirabelle_arith.ML@a564458f94db
child 73847 58f6b41efe88
permissions -rw-r--r--
reimplemented Mirabelle as Isabelle/ML presentation hook + Isabelle/Scala tool, but sledgehammer is still inactive;

(*  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