doc-src/TutorialI/Recdef/examples.thy
changeset 8771 026f37a86ea7
parent 8745 13b32661dde4
child 9541 d17c0b34d5c8
--- a/doc-src/TutorialI/Recdef/examples.thy	Sun Apr 23 11:41:45 2000 +0200
+++ b/doc-src/TutorialI/Recdef/examples.thy	Tue Apr 25 08:09:10 2000 +0200
@@ -14,7 +14,7 @@
 
 text{*\noindent
 The definition of \isa{fib} is accompanied by a \bfindex{measure function}
-\isa{\isasymlambda{}n.$\;$n} that maps the argument of \isa{fib} to a
+\isa{\isasymlambda{}n.$\;$n} which maps the argument of \isa{fib} to a
 natural number. The requirement is that in each equation the measure of the
 argument on the left-hand side is strictly greater than the measure of the
 argument of each recursive call. In the case of \isa{fib} this is
@@ -83,7 +83,7 @@
   "swap12 zs       = zs";
 
 text{*\noindent
-In the non-recursive case the termination measure degenerates to the empty
+For non-recursive functions the termination measure degenerates to the empty
 set \isa{\{\}}.
 *}