doc-src/TutorialI/Misc/simp.thy
changeset 11215 b44ad7e4c4d2
parent 11214 3b3cc0cf533f
child 11309 d666f11ca2d4
--- a/doc-src/TutorialI/Misc/simp.thy	Mon Mar 19 13:05:56 2001 +0100
+++ b/doc-src/TutorialI/Misc/simp.thy	Mon Mar 19 13:28:06 2001 +0100
@@ -135,7 +135,7 @@
 
 subsection{*Rewriting with Definitions*}
 
-text{*\index{simplification!with definitions}
+text{*\label{sec:Simp-with-Defs}\index{simplification!with definitions}
 Constant definitions (\S\ref{sec:ConstDefinitions}) can
 be used as simplification rules, but by default they are not.  Hence the
 simplifier does not expand them automatically, just as it should be:
@@ -237,7 +237,7 @@
 
 subsection{*Automatic Case Splits*}
 
-text{*\indexbold{case splits}\index{*split (method, attr.)|(}
+text{*\label{sec:AutoCaseSplits}\indexbold{case splits}\index{*split (method, attr.)|(}
 Goals containing @{text"if"}-expressions are usually proved by case
 distinction on the condition of the @{text"if"}. For example the goal
 *}