src/Pure/display_goal.ML
changeset 32168 116461b8fc01
parent 32167 d32817dda0e6
equal deleted inserted replaced
32167:d32817dda0e6 32168:116461b8fc01
    11   val show_consts: bool ref
    11   val show_consts: bool ref
    12   val pretty_flexpair: Proof.context -> term * term -> Pretty.T
    12   val pretty_flexpair: Proof.context -> term * term -> Pretty.T
    13   val pretty_goals: Proof.context -> {total: bool, main: bool, maxgoals: int} ->
    13   val pretty_goals: Proof.context -> {total: bool, main: bool, maxgoals: int} ->
    14     thm -> Pretty.T list
    14     thm -> Pretty.T list
    15   val pretty_goals_without_context: int -> thm -> Pretty.T list
    15   val pretty_goals_without_context: int -> thm -> Pretty.T list
    16   val print_goals_without_context: int -> thm -> unit
       
    17 end;
    16 end;
    18 
    17 
    19 structure Display_Goal: DISPLAY_GOAL =
    18 structure Display_Goal: DISPLAY_GOAL =
    20 struct
    19 struct
    21 
    20 
   117 
   116 
   118 fun pretty_goals_without_context n th =
   117 fun pretty_goals_without_context n th =
   119   pretty_goals (Syntax.init_pretty_global (Thm.theory_of_thm th))
   118   pretty_goals (Syntax.init_pretty_global (Thm.theory_of_thm th))
   120     {total = true, main = true, maxgoals = n} th;
   119     {total = true, main = true, maxgoals = n} th;
   121 
   120 
   122 val print_goals_without_context =
       
   123   (Pretty.writeln o Pretty.chunks) oo pretty_goals_without_context;
       
   124 
       
   125 end;
   121 end;
   126 
   122 
   127 end;
   123 end;
   128 
   124