tuned signature: more operations;
authorwenzelm
Wed, 26 Jul 2023 12:58:47 +0200
changeset 78465 4dffc47b7e91
parent 78464 12af46f2cd94
child 78466 1a68cd0c57d3
tuned signature: more operations;
src/HOL/Library/conditional_parametricity.ML
src/Pure/Isar/proof_display.ML
--- a/src/HOL/Library/conditional_parametricity.ML	Wed Jul 26 11:59:55 2023 +0200
+++ b/src/HOL/Library/conditional_parametricity.ML	Wed Jul 26 12:58:47 2023 +0200
@@ -502,7 +502,7 @@
     val thm = prove_goal settings lthy (SOME eq) goal;
     val (res, lthy') = Local_Theory.note (b, [thm]) lthy;
     val _ = if #suppress_print_theorem settings then () else
-      Proof_Display.print_results true (Position.thread_data ()) lthy' (("theorem",""), [res]);
+      Proof_Display.print_theorem (Position.thread_data ()) lthy' res;
   in
     (the_single (snd res), lthy')
   end;
--- a/src/Pure/Isar/proof_display.ML	Wed Jul 26 11:59:55 2023 +0200
+++ b/src/Pure/Isar/proof_display.ML	Wed Jul 26 12:58:47 2023 +0200
@@ -26,6 +26,7 @@
   val show_results: bool Config.T
   val print_results: bool -> Position.T -> Proof.context ->
     ((string * string) * (string * thm list) list) -> unit
+  val print_theorem: Position.T -> Proof.context -> string * thm list -> unit
   val print_consts: bool -> Position.T -> Proof.context ->
     (string * typ -> bool) -> (string * typ) list -> unit
   val markup_extern_label: Position.T -> (Markup.T * xstring) option
@@ -362,6 +363,9 @@
       | _ => Pretty.blk (1, [pretty_fact_name pos (kind, name), Pretty.fbrk,
           Pretty.blk (1, Pretty.str "(" :: pretty_facts ctxt facts @ [Pretty.str ")"])]));
 
+fun print_theorem pos ctxt fact =
+  print_results true pos ctxt ((Thm.theoremK, ""), [fact]);
+
 end;