doc-src/TutorialI/Datatype/Fundata.thy
changeset 8771 026f37a86ea7
parent 8745 13b32661dde4
child 9541 d17c0b34d5c8
--- a/doc-src/TutorialI/Datatype/Fundata.thy	Sun Apr 23 11:41:45 2000 +0200
+++ b/doc-src/TutorialI/Datatype/Fundata.thy	Tue Apr 25 08:09:10 2000 +0200
@@ -14,7 +14,7 @@
 term "Branch 0 (\\<lambda>i. Branch i (\\<lambda>n. Tip))";
 
 text{*\noindent of type \isa{(nat,nat)bigtree} is the tree whose
-root is labeled with 0 and whose $n$th subtree is labeled with $n$ and
+root is labeled with 0 and whose $i$th subtree is labeled with $i$ and
 has merely \isa{Tip}s as further subtrees.
 
 Function \isa{map_bt} applies a function to all labels in a \isa{bigtree}:
@@ -35,7 +35,7 @@
 
 The following lemma has a canonical proof  *}
 
-lemma "map_bt g (map_bt f T) = map_bt (g o f) T";
+lemma "map_bt (g o f) T = map_bt g (map_bt f T)";
 apply(induct_tac "T", auto).
 
 text{*\noindent