doc-src/IsarRef/Thy/Document_Preparation.thy
changeset 42669 04dfffda5671
parent 42658 8f5d5d71add0
child 42936 48a0a9db3453
equal deleted inserted replaced
42668:b98f22593f97 42669:04dfffda5671
   339   controls printing of implicit structures.
   339   controls printing of implicit structures.
   340 
   340 
   341   \item @{antiquotation_option_def show_abbrevs}~@{text "= bool"}
   341   \item @{antiquotation_option_def show_abbrevs}~@{text "= bool"}
   342   controls folding of abbreviations.
   342   controls folding of abbreviations.
   343 
   343 
   344   \item @{antiquotation_option_def long_names}~@{text "= bool"} forces
   344   \item @{antiquotation_option_def names_long}~@{text "= bool"} forces
   345   names of types and constants etc.\ to be printed in their fully
   345   names of types and constants etc.\ to be printed in their fully
   346   qualified internal form.
   346   qualified internal form.
   347 
   347 
   348   \item @{antiquotation_option_def short_names}~@{text "= bool"}
   348   \item @{antiquotation_option_def names_short}~@{text "= bool"}
   349   forces names of types and constants etc.\ to be printed unqualified.
   349   forces names of types and constants etc.\ to be printed unqualified.
   350   Note that internalizing the output again in the current context may
   350   Note that internalizing the output again in the current context may
   351   well yield a different result.
   351   well yield a different result.
   352 
   352 
   353   \item @{antiquotation_option_def unique_names}~@{text "= bool"}
   353   \item @{antiquotation_option_def names_unique}~@{text "= bool"}
   354   determines whether the printed version of qualified names should be
   354   determines whether the printed version of qualified names should be
   355   made sufficiently long to avoid overlap with names declared further
   355   made sufficiently long to avoid overlap with names declared further
   356   back.  Set to @{text false} for more concise output.
   356   back.  Set to @{text false} for more concise output.
   357 
   357 
   358   \item @{antiquotation_option_def eta_contract}~@{text "= bool"}
   358   \item @{antiquotation_option_def eta_contract}~@{text "= bool"}