src/Pure/goal_display.ML
changeset 51958 bca32217b304
parent 50543 42bbe637be54
child 51959 18d758e38d85
equal deleted inserted replaced
51953:ae755fd6c883 51958:bca32217b304
    18   val show_consts_raw: Config.raw
    18   val show_consts_raw: Config.raw
    19   val show_consts: bool Config.T
    19   val show_consts: bool Config.T
    20   val pretty_flexpair: Proof.context -> term * term -> Pretty.T
    20   val pretty_flexpair: Proof.context -> term * term -> Pretty.T
    21   val pretty_goals: Proof.context -> thm -> Pretty.T list
    21   val pretty_goals: Proof.context -> thm -> Pretty.T list
    22   val pretty_goals_without_context: thm -> Pretty.T list
    22   val pretty_goals_without_context: thm -> Pretty.T list
    23   val pretty_goal: {main: bool, limit: bool} -> Proof.context -> thm -> Pretty.T
    23   val pretty_goal: Proof.context -> thm -> Pretty.T
       
    24   val string_of_goal: Proof.context -> thm -> string
    24 end;
    25 end;
    25 
    26 
    26 structure Goal_Display: GOAL_DISPLAY =
    27 structure Goal_Display: GOAL_DISPLAY =
    27 struct
    28 struct
    28 
    29 
   146 fun pretty_goals_without_context th =
   147 fun pretty_goals_without_context th =
   147   let val ctxt =
   148   let val ctxt =
   148     Config.put show_main_goal true (Syntax.init_pretty_global (Thm.theory_of_thm th))
   149     Config.put show_main_goal true (Syntax.init_pretty_global (Thm.theory_of_thm th))
   149   in pretty_goals ctxt th end;
   150   in pretty_goals ctxt th end;
   150 
   151 
   151 fun pretty_goal {main, limit} ctxt th =
   152 fun pretty_goal ctxt th =
   152   Pretty.chunks (pretty_goals
   153   Pretty.chunks (pretty_goals (Config.put goals_total false ctxt) th);
   153     (ctxt
   154 
   154       |> Config.put show_main_goal main
   155 val string_of_goal = Pretty.string_of oo pretty_goal;
   155       |> not limit ? Config.put goals_limit (Thm.nprems_of th)
       
   156       |> Config.put goals_total false) th);
       
   157 
   156 
   158 end;
   157 end;
   159 
   158 
   160 end;
   159 end;
   161 
   160