src/Doc/ProgProve/Logic.thy
changeset 55361 d459a63ca42f
parent 55348 366718f2ff85
child 56116 bdc03e91684a
--- a/src/Doc/ProgProve/Logic.thy	Fri Feb 07 22:37:54 2014 +0100
+++ b/src/Doc/ProgProve/Logic.thy	Sat Feb 08 20:34:10 2014 +0100
@@ -496,7 +496,7 @@
 
 
 \section{Inductive Definitions}
-\label{sec:inductive-defs}\index{inductive definition}
+\label{sec:inductive-defs}\index{inductive definition|(}
 
 Inductive definitions are the third important definition facility, after
 datatypes and recursive function.
@@ -531,7 +531,7 @@
 @{text "ev 0 \<Longrightarrow> ev (0 + 2) \<Longrightarrow> ev((0 + 2) + 2) = ev 4"}
 \end{quote}
 
-\subsubsection{Rule Induction}
+\subsubsection{Rule Induction}\index{rule induction|(}
 
 Showing that all even numbers have some property is more complicated.  For
 example, let us prove that the inductive definition of even numbers agrees
@@ -753,7 +753,7 @@
 apply(metis step)
 done
 
-text{*
+text{*\index{rule induction|)}
 
 \subsection{The General Case}
 
@@ -787,8 +787,8 @@
 additional premises not involving @{text I}, so-called \conceptidx{side
 conditions}{side condition}. In rule inductions, these side conditions appear as additional
 assumptions. The \isacom{for} clause seen in the definition of the reflexive
-transitive closure merely simplifies the form of the induction rule.
-
+transitive closure simplifies the induction rule.
+\index{inductive definition|)}
 
 \subsection*{Exercises}