src/Doc/IsarRef/Inner_Syntax.thy
changeset 49699 1301ed115729
parent 48985 5386df44a037
child 50635 5543eff56b16
equal deleted inserted replaced
49698:f68e237e8c10 49699:1301ed115729
   124 
   124 
   125 subsection {* Details of printed content *}
   125 subsection {* Details of printed content *}
   126 
   126 
   127 text {*
   127 text {*
   128   \begin{tabular}{rcll}
   128   \begin{tabular}{rcll}
       
   129     @{attribute_def show_markup} & : & @{text attribute} \\
   129     @{attribute_def show_types} & : & @{text attribute} & default @{text false} \\
   130     @{attribute_def show_types} & : & @{text attribute} & default @{text false} \\
   130     @{attribute_def show_sorts} & : & @{text attribute} & default @{text false} \\
   131     @{attribute_def show_sorts} & : & @{text attribute} & default @{text false} \\
   131     @{attribute_def show_consts} & : & @{text attribute} & default @{text false} \\
   132     @{attribute_def show_consts} & : & @{text attribute} & default @{text false} \\
   132     @{attribute_def show_abbrevs} & : & @{text attribute} & default @{text true} \\
   133     @{attribute_def show_abbrevs} & : & @{text attribute} & default @{text true} \\
   133     @{attribute_def show_brackets} & : & @{text attribute} & default @{text false} \\
   134     @{attribute_def show_brackets} & : & @{text attribute} & default @{text false} \\
   147   is displayed for types, terms, theorems, goals etc.  See also
   148   is displayed for types, terms, theorems, goals etc.  See also
   148   \secref{sec:config}.
   149   \secref{sec:config}.
   149 
   150 
   150   \begin{description}
   151   \begin{description}
   151 
   152 
       
   153   \item @{attribute show_markup} controls direct inlining of markup
       
   154   into the printed representation of formal entities --- notably type
       
   155   and sort constraints.  This enables Prover IDE users to retrieve
       
   156   that information via tooltips or popups while hovering with the
       
   157   mouse over the output window, for example.  Consequently, this
       
   158   option is enabled by default for Isabelle/jEdit, but disabled for
       
   159   TTY and Proof~General~/Emacs where document markup would not work.
       
   160 
   152   \item @{attribute show_types} and @{attribute show_sorts} control
   161   \item @{attribute show_types} and @{attribute show_sorts} control
   153   printing of type constraints for term variables, and sort
   162   printing of type constraints for term variables, and sort
   154   constraints for type variables.  By default, neither of these are
   163   constraints for type variables.  By default, neither of these are
   155   shown in output.  If @{attribute show_sorts} is enabled, types are
   164   shown in output.  If @{attribute show_sorts} is enabled, types are
   156   always shown as well.
   165   always shown as well.  In Isabelle/jEdit, manual setting of these
       
   166   options is normally not required thanks to @{attribute show_markup}
       
   167   above.
   157 
   168 
   158   Note that displaying types and sorts may explain why a polymorphic
   169   Note that displaying types and sorts may explain why a polymorphic
   159   inference rule fails to resolve with some goal, or why a rewrite
   170   inference rule fails to resolve with some goal, or why a rewrite
   160   rule does not apply as expected.
   171   rule does not apply as expected.
   161 
   172