doc-src/LaTeXsugar/Sugar/Sugar.thy
changeset 33323 1932908057c7
parent 32898 e871d897969c
child 34877 ded5b770ec1c
equal deleted inserted replaced
33322:6ff4674499ca 33323:1932908057c7
   130 results in @{thm conjI[no_vars]}.
   130 results in @{thm conjI[no_vars]}.
   131 
   131 
   132 This \verb!no_vars! business can become a bit tedious.
   132 This \verb!no_vars! business can become a bit tedious.
   133 If you would rather never see question marks, simply put
   133 If you would rather never see question marks, simply put
   134 \begin{verbatim}
   134 \begin{verbatim}
   135 reset show_question_marks;
   135 show_question_marks := false;
   136 \end{verbatim}
   136 \end{verbatim}
   137 at the beginning of your file \texttt{ROOT.ML}.
   137 at the beginning of your file \texttt{ROOT.ML}.
   138 The rest of this document is produced with this flag reset.
   138 The rest of this document is produced with this flag set to \texttt{false}.
   139 
   139 
   140 Hint: Resetting \verb!show_question_marks! only suppresses question
   140 Hint: Setting \verb!show_question_marks! to \texttt{false} only
   141 marks; variables that end in digits, e.g. @{text"x1"}, are still
   141 suppresses question marks; variables that end in digits,
   142 printed with a trailing @{text".0"}, e.g. @{text"x1.0"}, their
   142 e.g. @{text"x1"}, are still printed with a trailing @{text".0"},
   143 internal index. This can be avoided by turning the last digit into a
   143 e.g. @{text"x1.0"}, their internal index. This can be avoided by
   144 subscript: write \verb!x\<^isub>1! and obtain the much nicer @{text"x\<^isub>1"}. *}
   144 turning the last digit into a subscript: write \verb!x\<^isub>1! and
   145 
   145 obtain the much nicer @{text"x\<^isub>1"}. *}
   146 (*<*)ML"Unsynchronized.reset show_question_marks"(*>*)
   146 
       
   147 (*<*)ML"show_question_marks := false"(*>*)
   147 
   148 
   148 subsection {*Qualified names*}
   149 subsection {*Qualified names*}
   149 
   150 
   150 text{* If there are multiple declarations of the same name, Isabelle prints
   151 text{* If there are multiple declarations of the same name, Isabelle prints
   151 the qualified name, for example @{text "T.length"}, where @{text T} is the
   152 the qualified name, for example @{text "T.length"}, where @{text T} is the
   413   \end{center}
   414   \end{center}
   414   is produced by the following code:
   415   is produced by the following code:
   415   \begin{quote}
   416   \begin{quote}
   416     \verb!\begin{center}!\\
   417     \verb!\begin{center}!\\
   417     \verb!\begin{tabular}{l@ {~~!\verb!@!\verb!{text "="}~~}l}!\\
   418     \verb!\begin{tabular}{l@ {~~!\verb!@!\verb!{text "="}~~}l}!\\
   418     \verb!@!\verb!{thm (lhs) foldl_Nil} & @!\verb!{thm (rhs) foldl_Nil}!\\
   419     \verb!@!\verb!{thm (lhs) foldl_Nil} & @!\verb!{thm (rhs) foldl_Nil}\\!\\
   419     \verb!@!\verb!{thm (lhs) foldl_Cons} & @!\verb!{thm (rhs) foldl_Cons}!\\
   420     \verb!@!\verb!{thm (lhs) foldl_Cons} & @!\verb!{thm (rhs) foldl_Cons}!\\
   420     \verb!\end{tabular}!\\
   421     \verb!\end{tabular}!\\
   421     \verb!\end{center}!
   422     \verb!\end{center}!
   422   \end{quote}
   423   \end{quote}
   423   Note the space between \verb!@! and \verb!{! in the tabular argument.
   424   Note the space between \verb!@! and \verb!{! in the tabular argument.
   428   (e.~g.~@{text "="}, @{text "\<equiv>"}, @{text "<"}).
   429   (e.~g.~@{text "="}, @{text "\<equiv>"}, @{text "<"}).
   429 
   430 
   430   Likewise, \verb!concl! may be used as a style to show just the
   431   Likewise, \verb!concl! may be used as a style to show just the
   431   conclusion of a proposition. For example, take \verb!hd_Cons_tl!:
   432   conclusion of a proposition. For example, take \verb!hd_Cons_tl!:
   432   \begin{center}
   433   \begin{center}
   433     @{thm [show_types] hd_Cons_tl}
   434     @{thm hd_Cons_tl}
   434   \end{center}
   435   \end{center}
   435   To print just the conclusion,
   436   To print just the conclusion,
   436   \begin{center}
   437   \begin{center}
   437     @{thm [show_types] (concl) hd_Cons_tl}
   438     @{thm (concl) hd_Cons_tl}
   438   \end{center}
   439   \end{center}
   439   type
   440   type
   440   \begin{quote}
   441   \begin{quote}
   441     \verb!\begin{center}!\\
   442     \verb!\begin{center}!\\
   442     \verb!@!\verb!{thm [show_types] (concl) hd_Cons_tl}!\\
   443     \verb!@!\verb!{thm (concl) hd_Cons_tl}!\\
   443     \verb!\end{center}!
   444     \verb!\end{center}!
   444   \end{quote}
   445   \end{quote}
   445   Beware that any options must be placed \emph{before}
   446   Beware that any options must be placed \emph{before}
   446   the style, as in this example.
   447   the style, as in this example.
   447 
   448