doc-src/Sledgehammer/sledgehammer.tex
changeset 42237 e645d7255bd4
parent 42234 7ec43598c8be
child 42442 036142bd0302
--- a/doc-src/Sledgehammer/sledgehammer.tex	Tue Apr 05 10:54:09 2011 +0200
+++ b/doc-src/Sledgehammer/sledgehammer.tex	Tue Apr 05 11:39:48 2011 +0200
@@ -564,21 +564,20 @@
 \item[$\bullet$] \textbf{\textit{tags}:} Each term (and subterm) is tagged with
 its type.
 
+\item[$\bullet$] \textbf{\textit{args}:} Constants are annotated with
+their type parameters, which are passed as extra arguments. This value is
+ignored if \textit{full\_types} is enabled.
+
 \item[$\bullet$] \textbf{\textit{mangled}:} Types are mangled in constant names.
 This value is available only if \textit{monomorphize} is enabled and
 \textit{full\_types} is disabled.
 
-\item[$\bullet$] \textbf{\textit{const\_args}:} Constants are annotated with
-their type parameters, which are passed as extra arguments. This value is
-ignored if \textit{full\_types} is enabled.
-
 \item[$\bullet$] \textbf{\textit{none}:} No type information is supplied to the
 ATP. This value is ignored if \textit{full\_types} is enabled.
 
-\item[$\bullet$] \textbf{\textit{smart}:} This is the same as
-\textit{tags} if \textit{full\_types} is enabled; otherwise, this is the
-same as \textit{mangled} if \textit{monomorphize} is enabled and
-\textit{const\_args} otherwise.
+\item[$\bullet$] \textbf{\textit{smart}:} If \textit{full\_types} is enabled,
+this is the same as \textit{tags}; otherwise, this is the
+same as \textit{args} otherwise.
 \end{enum}
 
 For SMT solvers, the type system is always \textit{mangled}.