src/Pure/more_thm.ML
changeset 69575 f77cc54f6d47
parent 68036 4c9e79aeadf0
child 70152 6218698851b9
equal deleted inserted replaced
69574:b4ea943ce0b7 69575:f77cc54f6d47
   113   val tag: string * string -> attribute
   113   val tag: string * string -> attribute
   114   val untag: string -> attribute
   114   val untag: string -> attribute
   115   val kind: string -> attribute
   115   val kind: string -> attribute
   116   val register_proofs: thm list lazy -> theory -> theory
   116   val register_proofs: thm list lazy -> theory -> theory
   117   val consolidate_theory: theory -> unit
   117   val consolidate_theory: theory -> unit
   118   val show_consts_raw: Config.raw
       
   119   val show_consts: bool Config.T
   118   val show_consts: bool Config.T
   120   val show_hyps_raw: Config.raw
       
   121   val show_hyps: bool Config.T
   119   val show_hyps: bool Config.T
   122   val show_tags_raw: Config.raw
       
   123   val show_tags: bool Config.T
   120   val show_tags: bool Config.T
   124   val pretty_flexpair: Proof.context -> term * term -> Pretty.T
   121   val pretty_flexpair: Proof.context -> term * term -> Pretty.T
   125   val pretty_thm_raw: Proof.context -> {quote: bool, show_hyps: bool} -> thm -> Pretty.T
   122   val pretty_thm_raw: Proof.context -> {quote: bool, show_hyps: bool} -> thm -> Pretty.T
   126   val pretty_thm: Proof.context -> thm -> Pretty.T
   123   val pretty_thm: Proof.context -> thm -> Pretty.T
   127   val pretty_thm_item: Proof.context -> thm -> Pretty.T
   124   val pretty_thm_item: Proof.context -> thm -> Pretty.T
   684 
   681 
   685 (** print theorems **)
   682 (** print theorems **)
   686 
   683 
   687 (* options *)
   684 (* options *)
   688 
   685 
   689 val show_consts_raw = Config.declare_option ("show_consts", \<^here>);
   686 val show_consts = Config.declare_option_bool ("show_consts", \<^here>);
   690 val show_consts = Config.bool show_consts_raw;
   687 val show_hyps = Config.declare_bool ("show_hyps", \<^here>) (K false);
   691 
   688 val show_tags = Config.declare_bool ("show_tags", \<^here>) (K false);
   692 val show_hyps_raw = Config.declare ("show_hyps", \<^here>) (fn _ => Config.Bool false);
       
   693 val show_hyps = Config.bool show_hyps_raw;
       
   694 
       
   695 val show_tags_raw = Config.declare ("show_tags", \<^here>) (fn _ => Config.Bool false);
       
   696 val show_tags = Config.bool show_tags_raw;
       
   697 
   689 
   698 
   690 
   699 (* pretty_thm etc. *)
   691 (* pretty_thm etc. *)
   700 
   692 
   701 fun pretty_tag (name, arg) = Pretty.strs [name, quote arg];
   693 fun pretty_tag (name, arg) = Pretty.strs [name, quote arg];