doc-src/IsarRef/Thy/Inner_Syntax.thy
changeset 42358 b47d41d9f4b5
parent 42279 6da43a5018e2
child 42596 6c621a9d612a
equal deleted inserted replaced
42357:3305f573294e 42358:b47d41d9f4b5
    98   \begin{mldecls} 
    98   \begin{mldecls} 
    99     @{index_ML show_types: "bool Config.T"} & default @{ML false} \\
    99     @{index_ML show_types: "bool Config.T"} & default @{ML false} \\
   100     @{index_ML show_sorts: "bool Config.T"} & default @{ML false} \\
   100     @{index_ML show_sorts: "bool Config.T"} & default @{ML false} \\
   101     @{index_ML show_consts: "bool Config.T"} & default @{ML false} \\
   101     @{index_ML show_consts: "bool Config.T"} & default @{ML false} \\
   102     @{index_ML show_abbrevs: "bool Config.T"} & default @{ML true} \\
   102     @{index_ML show_abbrevs: "bool Config.T"} & default @{ML true} \\
   103     @{index_ML long_names: "bool Unsynchronized.ref"} & default @{ML false} \\
       
   104     @{index_ML short_names: "bool Unsynchronized.ref"} & default @{ML false} \\
       
   105     @{index_ML unique_names: "bool Unsynchronized.ref"} & default @{ML true} \\
       
   106     @{index_ML show_brackets: "bool Config.T"} & default @{ML false} \\
   103     @{index_ML show_brackets: "bool Config.T"} & default @{ML false} \\
       
   104     @{index_ML Name_Space.long_names: "bool Config.T"} & default @{ML false} \\
       
   105     @{index_ML Name_Space.short_names: "bool Config.T"} & default @{ML false} \\
       
   106     @{index_ML Name_Space.unique_names: "bool Config.T"} & default @{ML true} \\
   107     @{index_ML eta_contract: "bool Config.T"} & default @{ML true} \\
   107     @{index_ML eta_contract: "bool Config.T"} & default @{ML true} \\
   108     @{index_ML Goal_Display.goals_limit: "int Config.T"} & default @{ML 10} \\
   108     @{index_ML Goal_Display.goals_limit: "int Config.T"} & default @{ML 10} \\
   109     @{index_ML Goal_Display.show_main_goal: "bool Config.T"} & default @{ML false} \\
   109     @{index_ML Goal_Display.show_main_goal: "bool Config.T"} & default @{ML false} \\
   110     @{index_ML show_hyps: "bool Config.T"} & default @{ML false} \\
   110     @{index_ML show_hyps: "bool Config.T"} & default @{ML false} \\
   111     @{index_ML show_tags: "bool Config.T"} & default @{ML false} \\
   111     @{index_ML show_tags: "bool Config.T"} & default @{ML false} \\
   142   Note that the output can be enormous, because polymorphic constants
   142   Note that the output can be enormous, because polymorphic constants
   143   often occur at several different type instances.
   143   often occur at several different type instances.
   144 
   144 
   145   \item @{ML show_abbrevs} controls folding of constant abbreviations.
   145   \item @{ML show_abbrevs} controls folding of constant abbreviations.
   146 
   146 
   147   \item @{ML long_names}, @{ML short_names}, and @{ML unique_names}
       
   148   control the way of printing fully qualified internal names in
       
   149   external form.  See also \secref{sec:antiq} for the document
       
   150   antiquotation options of the same names.
       
   151 
       
   152   \item @{ML show_brackets} controls bracketing in pretty printed
   147   \item @{ML show_brackets} controls bracketing in pretty printed
   153   output.  If set to @{ML true}, all sub-expressions of the pretty
   148   output.  If set to @{ML true}, all sub-expressions of the pretty
   154   printing tree will be parenthesized, even if this produces malformed
   149   printing tree will be parenthesized, even if this produces malformed
   155   term syntax!  This crude way of showing the internal structure of
   150   term syntax!  This crude way of showing the internal structure of
   156   pretty printed entities may occasionally help to diagnose problems
   151   pretty printed entities may occasionally help to diagnose problems
   157   with operator priorities, for example.
   152   with operator priorities, for example.
       
   153 
       
   154   \item @{ML Name_Space.long_names}, @{ML Name_Space.short_names}, and
       
   155   @{ML Name_Space.unique_names} control the way of printing fully
       
   156   qualified internal names in external form.  See also
       
   157   \secref{sec:antiq} for the document antiquotation options of the
       
   158   same names.
   158 
   159 
   159   \item @{ML eta_contract} controls @{text "\<eta>"}-contracted printing of
   160   \item @{ML eta_contract} controls @{text "\<eta>"}-contracted printing of
   160   terms.
   161   terms.
   161 
   162 
   162   The @{text \<eta>}-contraction law asserts @{prop "(\<lambda>x. f x) \<equiv> f"},
   163   The @{text \<eta>}-contraction law asserts @{prop "(\<lambda>x. f x) \<equiv> f"},