src/HOL/Mirabelle/Tools/mirabelle_arith.ML
author boehmes
Wed, 02 Sep 2009 21:31:58 +0200
changeset 32498 1132c7c13f36
parent 32496 4ab00a2642c3
child 32515 e7c0d3c0494a
permissions -rw-r--r--
Mirabelle: actions are responsible for handling exceptions, Mirabelle core logs only structural information, measuring running times for sledgehammer and subsequent metis invocation, Mirabelle produces reports for every theory (only for sledgehammer at the moment)

(* Title:  mirabelle_arith.ML
   Author: Jasmin Blanchette and Sascha Boehme
*)

structure Mirabelle_Arith : MIRABELLE_ACTION =
struct

fun arith_action {pre, timeout, log, ...} =
  if Mirabelle.can_apply timeout Arith_Data.arith_tac pre
  then log "arith: succeeded"
  else ()
  handle TimeLimit.TimeOut => log "arith: time out"

fun invoke _ = Mirabelle.register ("arith", arith_action)

end