src/Pure/Tools/find_theorems.ML
changeset 30186 1f836e949ac2
parent 30143 98a986b02022
child 30188 82144a95f9ec
--- a/src/Pure/Tools/find_theorems.ML	Sun Mar 01 14:36:27 2009 +0100
+++ b/src/Pure/Tools/find_theorems.ML	Sun Mar 01 14:45:23 2009 +0100
@@ -6,16 +6,14 @@
 
 signature FIND_THEOREMS =
 sig
-  val limit: int ref
-  val tac_limit: int ref
-
   datatype 'term criterion =
     Name of string | Intro | Elim | Dest | Solves | Simp of 'term |
     Pattern of 'term
-
+  val tac_limit: int ref
+  val limit: int ref
   val find_theorems: Proof.context -> thm option -> bool ->
     (bool * string criterion) list -> (Facts.ref * thm) list
-
+  val pretty_thm: Proof.context -> Facts.ref * thm -> Pretty.T
   val print_theorems: Proof.context -> thm option -> int option -> bool ->
     (bool * string criterion) list -> unit
 end;
@@ -344,8 +342,7 @@
 
 fun find_theorems ctxt opt_goal rem_dups raw_criteria =
   let
-    val add_prems = Seq.hd o (TRY (Method.insert_tac
-                                     (Assumption.prems_of ctxt) 1));
+    val add_prems = Seq.hd o (TRY (Method.insert_tac (Assumption.prems_of ctxt) 1));
     val opt_goal' = Option.map add_prems opt_goal;
 
     val criteria = map (apsnd (read_criterion ctxt)) raw_criteria;
@@ -359,6 +356,11 @@
       else raw_matches;
   in matches end;
 
+
+fun pretty_thm ctxt (thmref, thm) = Pretty.block
+  [Pretty.str (Facts.string_of_ref thmref), Pretty.str ":", Pretty.brk 1,
+    ProofContext.pretty_thm ctxt thm];
+
 fun print_theorems ctxt opt_goal opt_limit rem_dups raw_criteria =
   let
     val start = start_timing ();
@@ -382,7 +384,7 @@
           (if len <= lim then ""
            else " (" ^ string_of_int lim ^ " displayed)")
            ^ end_msg ^ ":"), Pretty.str ""] @
-        map Display.pretty_fact thms)
+        map (pretty_thm ctxt) thms)
     |> Pretty.chunks |> Pretty.writeln
   end;