src/HOL/Tools/SMT/smt_config.ML
changeset 46736 4dc7ddb47350
parent 46042 ab32a87ba01a
child 46949 94aa7b81bcf6
--- a/src/HOL/Tools/SMT/smt_config.ML	Tue Feb 28 21:58:59 2012 +0100
+++ b/src/HOL/Tools/SMT/smt_config.ML	Wed Feb 29 17:43:41 2012 +0100
@@ -14,6 +14,7 @@
     options: Proof.context -> string list }
   val add_solver: solver_info -> Context.generic -> Context.generic
   val set_solver_options: string * string -> Context.generic -> Context.generic
+  val is_available: Proof.context -> string -> bool
   val available_solvers_of: Proof.context -> string list
   val select_solver: string -> Context.generic -> Context.generic
   val solver_of: Proof.context -> string