doc-src/TutorialI/Advanced/simp.thy
changeset 10845 3696bc935bbd
parent 10795 9e888d60d3e5
child 10885 90695f46440b
--- a/doc-src/TutorialI/Advanced/simp.thy	Wed Jan 10 11:07:11 2001 +0100
+++ b/doc-src/TutorialI/Advanced/simp.thy	Wed Jan 10 11:08:29 2001 +0100
@@ -157,7 +157,7 @@
 
 subsubsection{*The preprocessor*}
 
-text{*
+text{*\label{sec:simp-preprocessor}
 When some theorem is declared a simplification rule, it need not be a
 conditional equation already.  The simplifier will turn it into a set of
 conditional equations automatically.  For example, given @{prop"f x =
@@ -175,7 +175,8 @@
 \end{eqnarray}
 Once this conversion process is finished, all remaining non-equations
 $P$ are turned into trivial equations $P = True$.
-For example, the formula @{prop"(p \<longrightarrow> q \<and> r) \<and> s"} is converted into the three rules
+For example, the formula \begin{center}@{prop"(p \<longrightarrow> q \<and> r) \<and> s"}\end{center}
+is converted into the three rules
 \begin{center}
 @{prop"p \<Longrightarrow> q = True"},\quad  @{prop"p \<Longrightarrow> r = True"},\quad  @{prop"s = True"}.
 \end{center}