doc-src/Ref/simplifier.tex
changeset 16019 0e1405402d53
parent 15027 d23887300b96
child 30184 37969710e61f
--- a/doc-src/Ref/simplifier.tex	Sun May 22 16:51:06 2005 +0200
+++ b/doc-src/Ref/simplifier.tex	Sun May 22 16:51:07 2005 +0200
@@ -1224,12 +1224,10 @@
 first-order logic; the code is largely taken from {\tt FOL/simpdata.ML} of the
 Isabelle sources.
 
-The simplifier and the case splitting tactic, which reside on separate files,
-are not part of Pure Isabelle.  They must be loaded explicitly by the
-object-logic as follows (below \texttt{\~\relax\~\relax} refers to
-\texttt{\$ISABELLE_HOME}):
+The case splitting tactic, which resides on a separate files, is not part of
+Pure Isabelle.  It needs to be loaded explicitly by the object-logic as
+follows (below \texttt{\~\relax\~\relax} refers to \texttt{\$ISABELLE_HOME}):
 \begin{ttbox}
-use "\~\relax\~\relax/src/Provers/simplifier.ML";
 use "\~\relax\~\relax/src/Provers/splitter.ML";
 \end{ttbox}
 
@@ -1461,23 +1459,6 @@
 \end{ttbox}
 
 
-\subsection{Theory setup}\index{simplification!setting up the theory}
-\begin{ttbox}\indexbold{*Simplifier.setup}\index{*setup!simplifier}
-Simplifier.setup: (theory -> theory) list
-\end{ttbox}
-
-Advanced theory related features of the simplifier (e.g.\ implicit
-simpset support) have to be set up explicitly.  The simplifier already
-provides a suitable setup function definition.  This has to be
-installed into the base theory of any new object-logic via a
-\texttt{setup} declaration.
-
-For example, this is done in \texttt{FOL/IFOL.thy} as follows:
-\begin{ttbox}
-setup Simplifier.setup
-\end{ttbox}
-
-
 \index{simplification|)}