minor doc fixes
authorblanchet
Sun, 01 May 2011 18:57:45 +0200
changeset 42591 f139d0ac2d44
parent 42590 03834570af86
child 42592 fa2cf11d6351
child 42596 6c621a9d612a
minor doc fixes
doc-src/Sledgehammer/sledgehammer.tex
--- a/doc-src/Sledgehammer/sledgehammer.tex	Sun May 01 18:52:38 2011 +0200
+++ b/doc-src/Sledgehammer/sledgehammer.tex	Sun May 01 18:57:45 2011 +0200
@@ -573,10 +573,10 @@
 \begin{enum}
 \item[$\bullet$] \textbf{\textit{many\_typed}:} Use the prover's support for
 many-typed first-order logic if available; otherwise, fall back on
-\textit{mangled}. The problem is monomorphized, meaning that the problem's type
-variables are instantiated with heuristically chosen ground types.
-Monomorphization can simplify reasoning but also leads to larger fact bases,
-which can slow down the ATPs.
+\textit{mangled\_preds}. The problem is monomorphized, meaning that the
+problem's type variables are instantiated with heuristically chosen ground
+types. Monomorphization can simplify reasoning but also leads to larger fact
+bases, which can slow down the ATPs.
 
 \item[$\bullet$] \textbf{\textit{preds}:} Types are encoded using a binary predicate
 $\mathit{has\_type\/}(\tau, t)$ that restricts the range of bound variables.
@@ -628,7 +628,7 @@
 \textit{tags}?,
 \textit{mono\_tags}?,
 \textit{mangled\_tags}?:} \\
-If the exclamation mark (!) is replaced by an question mark (?), the type
+If the exclamation mark (!)\ is replaced by an question mark (?),\ the type
 systems type only nonmonotonic (and hence especially dangerous) types. Not
 implemented yet.
 
@@ -650,7 +650,8 @@
 \opdefault{monomorphize\_limit}{int}{\upshape 4}
 Specifies the maximum number of iterations for the monomorphization fixpoint
 construction. The higher this limit is, the more monomorphic instances are
-potentially generated.
+potentially generated. Whether monomorphization takes place depends on the
+type system used.
 \end{enum}
 
 \subsection{Relevance Filter}