doc-src/LaTeXsugar/Sugar/Sugar.thy
changeset 38980 af73cf0dc31f
parent 38798 89f273ab1d42
child 41413 64cd30d6b0b8
--- a/doc-src/LaTeXsugar/Sugar/Sugar.thy	Wed Sep 01 23:43:45 2010 +0200
+++ b/doc-src/LaTeXsugar/Sugar/Sugar.thy	Thu Sep 02 00:48:07 2010 +0200
@@ -132,19 +132,19 @@
 This \verb!no_vars! business can become a bit tedious.
 If you would rather never see question marks, simply put
 \begin{quote}
-@{ML "show_question_marks := false"}\verb!;!
+@{ML "show_question_marks_default := false"}\verb!;!
 \end{quote}
 at the beginning of your file \texttt{ROOT.ML}.
 The rest of this document is produced with this flag set to \texttt{false}.
 
-Hint: Setting \verb!show_question_marks! to \texttt{false} only
+Hint: Setting \verb!show_question_marks_default! to \texttt{false} only
 suppresses question marks; variables that end in digits,
 e.g. @{text"x1"}, are still printed with a trailing @{text".0"},
 e.g. @{text"x1.0"}, their internal index. This can be avoided by
 turning the last digit into a subscript: write \verb!x\<^isub>1! and
 obtain the much nicer @{text"x\<^isub>1"}. *}
 
-(*<*)ML "show_question_marks := false"(*>*)
+(*<*)declare [[show_question_marks = false]](*>*)
 
 subsection {*Qualified names*}