doc-src/TutorialI/ToyList/ToyList.thy
changeset 9494 44fefb6e9994
parent 9458 c613cd06d5cf
child 9541 d17c0b34d5c8
--- a/doc-src/TutorialI/ToyList/ToyList.thy	Wed Aug 02 11:30:38 2000 +0200
+++ b/doc-src/TutorialI/ToyList/ToyList.thy	Wed Aug 02 13:17:11 2000 +0200
@@ -220,8 +220,9 @@
 text{*
 \subsubsection*{First lemma: \texttt{rev(xs \at~ys) = (rev ys) \at~(rev xs)}}
 
-After abandoning the above proof attempt\indexbold{abandon proof} (at the shell level type
-\isacommand{oops}) we start a new proof:
+After abandoning the above proof attempt\indexbold{abandon
+proof}\indexbold{proof!abandon} (at the shell level type
+\isacommand{oops}\indexbold{*oops}) we start a new proof:
 *}
 
 lemma rev_app [simp]: "rev(xs @ ys) = (rev ys) @ (rev xs)";