diff -r 279da0358aa9 -r 09a6c44a48ea doc-src/TutorialI/Recdef/examples.thy --- a/doc-src/TutorialI/Recdef/examples.thy Thu Jul 26 18:23:38 2001 +0200 +++ b/doc-src/TutorialI/Recdef/examples.thy Fri Aug 03 18:04:55 2001 +0200 @@ -3,7 +3,7 @@ (*>*) text{* -Here is a simple example, the Fibonacci function: +Here is a simple example, the \rmindex{Fibonacci function}: *} consts fib :: "nat \ nat"; @@ -13,7 +13,8 @@ "fib (Suc(Suc x)) = fib x + fib (Suc x)"; text{*\noindent -The definition of @{term"fib"} is accompanied by a \bfindex{measure function} +\index{measure functions}% +The definition of @{term"fib"} is accompanied by a \textbf{measure function} @{term"%n. n"} which maps the argument of @{term"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 @@ -38,7 +39,8 @@ The details of tupled $\lambda$-abstractions @{text"\(x\<^sub>1,\,x\<^sub>n)"} are explained in \S\ref{sec:products}, but for now your intuition is all you need. -Pattern matching need not be exhaustive: +Pattern matching\index{pattern matching!and \isacommand{recdef}} +need not be exhaustive: *} consts last :: "'a list \ 'a";