--- a/doc-src/TutorialI/Advanced/WFrec.thy Fri Jan 12 16:28:14 2001 +0100
+++ b/doc-src/TutorialI/Advanced/WFrec.thy Fri Jan 12 16:32:01 2001 +0100
@@ -28,11 +28,11 @@
left-hand side of an equation and $r$ the argument of some recursive call on
the corresponding right-hand side, induces a well-founded relation. For a
systematic account of termination proofs via well-founded relations see, for
-example, \cite{Baader-Nipkow}.
+example, Baader and Nipkow~\cite{Baader-Nipkow}.
Each \isacommand{recdef} definition should be accompanied (after the name of
the function) by a well-founded relation on the argument type of the
-function. The HOL library formalizes some of the most important
+function. HOL formalizes some of the most important
constructions of well-founded relations (see \S\ref{sec:Well-founded}). For
example, @{term"measure f"} is always well-founded, and the lexicographic
product of two well-founded relations is again well-founded, which we relied
@@ -50,7 +50,7 @@
text{*
Lexicographic products of measure functions already go a long
-way. Furthermore you may embed some type in an
+way. Furthermore, you may embed a type in an
existing well-founded relation via the inverse image construction @{term
inv_image}. All these constructions are known to \isacommand{recdef}. Thus you
will never have to prove well-foundedness of any relation composed