src/HOL/Tools/Mirabelle/mirabelle_presburger.ML
author wenzelm
Tue, 16 Nov 2021 21:43:41 +0100
changeset 74799 3dfb8e47a6b7
parent 74516 2c093a3167d1
child 74948 15ce207f69c8
permissions -rw-r--r--
removed redundant test (see also 86fac52c2795, a9fea3f11cc0);

(*  Title:      HOL/Mirabelle/Tools/mirabelle_presburger.ML
    Author:     Martin Desharnais, MPI-INF Saarbrücken

Mirabelle action: "presburger".
*)

structure Mirabelle_Presburger: MIRABELLE_ACTION =
struct

fun make_action ({timeout, ...} : Mirabelle.action_context) =
  let
    val _ = Timing.timing
    fun run_action ({pre, ...} : Mirabelle.command) =
      (case Timing.timing (Mirabelle.can_apply timeout (Cooper.tac true [] [])) pre of
        ({cpu, ...}, true) => "succeeded (" ^ Time.toString cpu ^ " s)"
      | (_, false) => "failed")
  in {run_action = run_action, finalize = K ""} end

val () = Mirabelle.register_action "presburger" make_action

end