doc-src/TutorialI/Trie/Trie.thy
changeset 9541 d17c0b34d5c8
parent 9458 c613cd06d5cf
child 9689 751fde5307e4
--- a/doc-src/TutorialI/Trie/Trie.thy	Fri Aug 04 23:02:11 2000 +0200
+++ b/doc-src/TutorialI/Trie/Trie.thy	Sun Aug 06 15:26:53 2000 +0200
@@ -81,8 +81,8 @@
 options:
 *};
 
-theorems [simp] = Let_def;
-theorems [split] = option.split;
+lemmas [simp] = Let_def;
+lemmas [split] = option.split;
 
 text{*\noindent
 The reason becomes clear when looking (probably after a failed proof
@@ -105,7 +105,6 @@
 \isa{as} is instantiated.
 The start of the proof is completely conventional:
 *};
-
 apply(induct_tac as, auto);
 
 txt{*\noindent
@@ -119,15 +118,13 @@
 well now. It turns out that instead of induction, case distinction
 suffices:
 *};
-
-apply(case_tac[!] bs);
-by(auto);
+by(case_tac[!] bs, auto);
 
 text{*\noindent
-Both \isaindex{case_tac} and \isaindex{induct_tac}
-take an optional first argument that specifies the range of subgoals they are
-applied to, where \isa{!} means all subgoals, i.e.\ \isa{[1-3]} in our case. Individual
-subgoal numbers are also allowed.
+All methods ending in \isa{tac} take an optional first argument that
+specifies the range of subgoals they are applied to, where \isa{[!]} means all
+subgoals, i.e.\ \isa{[1-3]} in our case. Individual subgoal numbers,
+e.g. \isa{[2]} are also allowed.
 
 This proof may look surprisingly straightforward. However, note that this
 comes at a cost: the proof script is unreadable because the