src/Pure/Isar/proof_display.ML
author wenzelm
Thu, 23 Jul 2009 16:52:16 +0200
changeset 32145 220c9e439d39
parent 32091 30e2ffbba718
child 33389 bb3a5fa94a91
permissions -rw-r--r--
clarified pretty_goals, pretty_thm_aux: plain context; explicit pretty_goals_without_context, print_goals_without_context; tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/Isar/proof_display.ML
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     2
    Author:     Makarius
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     3
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
     4
Printing of theorems, goals, results etc.
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     5
*)
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     6
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     7
signature PROOF_DISPLAY =
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
     8
sig
30628
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
     9
  val pp_context: Proof.context -> Pretty.T
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    10
  val pp_thm: thm -> Pretty.T
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    11
  val pp_typ: theory -> typ -> Pretty.T
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    12
  val pp_term: theory -> term -> Pretty.T
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    13
  val pp_ctyp: ctyp -> Pretty.T
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    14
  val pp_cterm: cterm -> Pretty.T
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    15
  val print_theorems_diff: theory -> theory -> unit
28092
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    16
  val print_theorems: theory -> unit
22335
6c4204df6863 pretty_full_theory: expose in signature.
aspinall
parents: 22095
diff changeset
    17
  val pretty_full_theory: bool -> theory -> Pretty.T
28092
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    18
  val print_theory: theory -> unit
20311
3666316adad6 moved debug option to proof_display.ML (again);
wenzelm
parents: 20253
diff changeset
    19
  val string_of_rule: Proof.context -> string -> thm -> string
27857
fdf43ffceae0 removed obsolete present_results;
wenzelm
parents: 27176
diff changeset
    20
  val print_results: bool -> Proof.context -> ((string * string) * (string * thm list) list) -> unit
fdf43ffceae0 removed obsolete present_results;
wenzelm
parents: 27176
diff changeset
    21
  val pretty_consts: Proof.context -> (string * typ -> bool) -> (string * typ) list -> Pretty.T
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    22
end
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    23
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    24
structure ProofDisplay: PROOF_DISPLAY =
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    25
struct
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    26
20235
3cbf73ed92f8 ProofContext.legacy_pretty_thm;
wenzelm
parents: 20211
diff changeset
    27
(* toplevel pretty printing *)
20211
c7f907f41f7c moved pprint functions to Isar/proof_display.ML;
wenzelm
parents: 19482
diff changeset
    28
30628
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    29
fun pp_context ctxt =
20311
3666316adad6 moved debug option to proof_display.ML (again);
wenzelm
parents: 20253
diff changeset
    30
 (if ! ProofContext.debug then
20211
c7f907f41f7c moved pprint functions to Isar/proof_display.ML;
wenzelm
parents: 19482
diff changeset
    31
    Pretty.quote (Pretty.big_list "proof context:" (ProofContext.pretty_context ctxt))
c7f907f41f7c moved pprint functions to Isar/proof_display.ML;
wenzelm
parents: 19482
diff changeset
    32
  else Pretty.str "<context>");
c7f907f41f7c moved pprint functions to Isar/proof_display.ML;
wenzelm
parents: 19482
diff changeset
    33
30628
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    34
fun pp_thm th =
30724
2e54e89bcce7 pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
wenzelm
parents: 30628
diff changeset
    35
  let
2e54e89bcce7 pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
wenzelm
parents: 30628
diff changeset
    36
    val thy = Thm.theory_of_thm th;
2e54e89bcce7 pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
wenzelm
parents: 30628
diff changeset
    37
    val flags = {quote = true, show_hyps = false, show_status = true};
32145
220c9e439d39 clarified pretty_goals, pretty_thm_aux: plain context;
wenzelm
parents: 32091
diff changeset
    38
  in Display.pretty_thm_raw (Syntax.init_pretty_global thy) flags th end;
20211
c7f907f41f7c moved pprint functions to Isar/proof_display.ML;
wenzelm
parents: 19482
diff changeset
    39
30628
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    40
val pp_typ = Pretty.quote oo Syntax.pretty_typ_global;
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    41
val pp_term = Pretty.quote oo Syntax.pretty_term_global;
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    42
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    43
fun pp_ctyp cT = pp_typ (Thm.theory_of_ctyp cT) (Thm.typ_of cT);
4078276bcace removed obsolete pprint operations;
wenzelm
parents: 30364
diff changeset
    44
fun pp_cterm ct = pp_term (Thm.theory_of_cterm ct) (Thm.term_of ct);
20211
c7f907f41f7c moved pprint functions to Isar/proof_display.ML;
wenzelm
parents: 19482
diff changeset
    45
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    46
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    47
(* theorems and theory *)
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    48
27176
3735b80d06fc Facts.dest/export_static: content difference;
wenzelm
parents: 26949
diff changeset
    49
fun pretty_theorems_diff prev_thys thy =
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    50
  let
27176
3735b80d06fc Facts.dest/export_static: content difference;
wenzelm
parents: 26949
diff changeset
    51
    val pretty_fact = ProofContext.pretty_fact (ProofContext.init thy);
28210
c164d1892553 more procise printing of fact names;
wenzelm
parents: 28092
diff changeset
    52
    val thmss = Facts.dest_static (map PureThy.facts_of prev_thys) (PureThy.facts_of thy);
c164d1892553 more procise printing of fact names;
wenzelm
parents: 28092
diff changeset
    53
  in Pretty.big_list "theorems:" (map #1 (sort_wrt (#1 o #2) (map (`pretty_fact) thmss))) end;
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    54
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    55
fun print_theorems_diff prev_thy thy =
27176
3735b80d06fc Facts.dest/export_static: content difference;
wenzelm
parents: 26949
diff changeset
    56
  Pretty.writeln (pretty_theorems_diff [prev_thy] thy);
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    57
27176
3735b80d06fc Facts.dest/export_static: content difference;
wenzelm
parents: 26949
diff changeset
    58
fun pretty_theorems thy = pretty_theorems_diff (Theory.parents_of thy) thy;
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    59
val print_theorems = Pretty.writeln o pretty_theorems;
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    60
22872
d7189dc8939c tuned ProofDisplay.pretty_full_theory;
wenzelm
parents: 22335
diff changeset
    61
fun pretty_full_theory verbose thy =
d7189dc8939c tuned ProofDisplay.pretty_full_theory;
wenzelm
parents: 22335
diff changeset
    62
  Pretty.chunks (Display.pretty_full_theory verbose thy @ [pretty_theorems thy]);
20621
29d57880ba00 'print_theory': bang option for full verbosity;
wenzelm
parents: 20311
diff changeset
    63
22872
d7189dc8939c tuned ProofDisplay.pretty_full_theory;
wenzelm
parents: 22335
diff changeset
    64
val print_theory = Pretty.writeln o pretty_full_theory false;
22335
6c4204df6863 pretty_full_theory: expose in signature.
aspinall
parents: 22095
diff changeset
    65
19432
cae7cc072994 added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
wenzelm
parents: 18799
diff changeset
    66
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    67
(* refinement rule *)
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    68
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    69
fun pretty_rule ctxt s thm =
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    70
  Pretty.block [Pretty.str (s ^ " attempt to solve goal by exported rule:"),
32091
30e2ffbba718 proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents: 30724
diff changeset
    71
    Pretty.fbrk, Display.pretty_thm_aux ctxt false thm];
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    72
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    73
val string_of_rule = Pretty.string_of ooo pretty_rule;
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    74
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    75
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    76
(* results *)
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    77
28092
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    78
local
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    79
28087
a9cccdd9d521 pretty_fact/results: display base only, since results now come with full names (note that Facts.extern is not really well-defined unless we present the real target context);
wenzelm
parents: 27857
diff changeset
    80
fun pretty_fact_name (kind, "") = Pretty.str kind
a9cccdd9d521 pretty_fact/results: display base only, since results now come with full names (note that Facts.extern is not really well-defined unless we present the real target context);
wenzelm
parents: 27857
diff changeset
    81
  | pretty_fact_name (kind, name) = Pretty.block [Pretty.str kind, Pretty.brk 1,
30364
577edc39b501 moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents: 30280
diff changeset
    82
      Pretty.str (Long_Name.base_name name), Pretty.str ":"];
28087
a9cccdd9d521 pretty_fact/results: display base only, since results now come with full names (note that Facts.extern is not really well-defined unless we present the real target context);
wenzelm
parents: 27857
diff changeset
    83
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    84
fun pretty_facts ctxt =
19482
9f11af8f7ef9 tuned basic list operators (flat, maps, map_filter);
wenzelm
parents: 19432
diff changeset
    85
  flat o (separate [Pretty.fbrk, Pretty.str "and "]) o
30724
2e54e89bcce7 pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
wenzelm
parents: 30628
diff changeset
    86
    map (single o ProofContext.pretty_fact_aux ctxt false);
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
    87
27857
fdf43ffceae0 removed obsolete present_results;
wenzelm
parents: 27176
diff changeset
    88
in
fdf43ffceae0 removed obsolete present_results;
wenzelm
parents: 27176
diff changeset
    89
28092
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    90
fun print_results do_print ctxt ((kind, name), facts) =
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    91
  if not do_print orelse kind = "" orelse kind = Thm.internalK then ()
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    92
  else if name = "" then
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    93
    Pretty.writeln (Pretty.block (Pretty.str kind :: Pretty.brk 1 :: pretty_facts ctxt facts))
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    94
  else Pretty.writeln
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    95
    (case facts of
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    96
      [fact] => Pretty.blk (1, [pretty_fact_name (kind, name), Pretty.fbrk,
30724
2e54e89bcce7 pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
wenzelm
parents: 30628
diff changeset
    97
        ProofContext.pretty_fact_aux ctxt false fact])
28092
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    98
    | _ => Pretty.blk (1, [pretty_fact_name (kind, name), Pretty.fbrk,
5886e9359aa8 no pervasive bindings;
wenzelm
parents: 28087
diff changeset
    99
        Pretty.blk (1, Pretty.str "(" :: pretty_facts ctxt facts @ [Pretty.str ")"])]));
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
   100
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
   101
end;
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
   102
20889
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   103
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   104
(* consts *)
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   105
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   106
local
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   107
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   108
fun pretty_var ctxt (x, T) =
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   109
  Pretty.block [Pretty.str x, Pretty.str " ::", Pretty.brk 1,
24920
2a45e400fdad generic Syntax.pretty/string_of operations;
wenzelm
parents: 22872
diff changeset
   110
    Pretty.quote (Syntax.pretty_typ ctxt T)];
20889
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   111
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   112
fun pretty_vars ctxt kind vs = Pretty.big_list kind (map (pretty_var ctxt) vs);
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   113
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   114
in
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   115
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   116
fun pretty_consts ctxt pred cs =
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   117
  (case filter pred (#1 (ProofContext.inferred_fixes ctxt)) of
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   118
    [] => pretty_vars ctxt "constants" cs
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   119
  | ps => Pretty.chunks [pretty_vars ctxt "parameters" ps, pretty_vars ctxt "constants" cs]);
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   120
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   121
end;
f625a65bfed5 added pretty_consts (from specification.ML);
wenzelm
parents: 20621
diff changeset
   122
17369
dec2ddbb3edf Printing of Isar proof elements etc.
wenzelm
parents:
diff changeset
   123
end;