src/HOL/Tools/Metis/metis_reconstruct.ML
changeset 40665 1a65f0c74827
parent 40264 b91e2e16d994
child 40724 d01a1b3ab23d
--- a/src/HOL/Tools/Metis/metis_reconstruct.ML	Mon Nov 22 23:37:00 2010 +0100
+++ b/src/HOL/Tools/Metis/metis_reconstruct.ML	Tue Nov 23 18:26:56 2010 +0100
@@ -13,6 +13,8 @@
 
   val trace : bool Config.T
   val trace_msg : Proof.context -> (unit -> string) -> unit
+  val verbose : bool Config.T
+  val verbose_warning : Proof.context -> string -> unit
   val lookth : (Metis_Thm.thm * 'a) list -> Metis_Thm.thm -> 'a
   val untyped_aconv : term -> term -> bool
   val replay_one_inference :
@@ -30,8 +32,11 @@
 open Metis_Translate
 
 val (trace, trace_setup) = Attrib.config_bool "trace_metis" (K false)
+val (verbose, verbose_setup) = Attrib.config_bool "verbose_metis" (K true)
 
 fun trace_msg ctxt msg = if Config.get ctxt trace then tracing (msg ()) else ()
+fun verbose_warning ctxt msg =
+  if Config.get ctxt verbose then warning msg else ()
 
 datatype term_or_type = SomeTerm of term | SomeType of typ
 
@@ -821,6 +826,6 @@
                     \Error when discharging Skolem assumptions.")
     end
 
-val setup = trace_setup
+val setup = trace_setup #> verbose_setup
 
 end;