doc-src/TutorialI/Trie/Trie.thy
changeset 10795 9e888d60d3e5
parent 10171 59d6633835fa
child 10971 6852682eaf16
--- a/doc-src/TutorialI/Trie/Trie.thy	Fri Jan 05 18:32:33 2001 +0100
+++ b/doc-src/TutorialI/Trie/Trie.thy	Fri Jan 05 18:32:57 2001 +0100
@@ -3,7 +3,7 @@
 (*>*)
 text{*
 To minimize running time, each node of a trie should contain an array that maps
-letters to subtries. We have chosen a (sometimes) more space efficient
+letters to subtries. We have chosen a
 representation where the subtries are held in an association list, i.e.\ a
 list of (letter,trie) pairs.  Abstracting over the alphabet @{typ"'a"} and the
 values @{typ"'v"} we define a trie as follows:
@@ -67,7 +67,7 @@
   "update t (a#as) v =
      (let tt = (case assoc (alist t) a of
                   None \<Rightarrow> Trie None [] | Some at \<Rightarrow> at)
-      in Trie (value t) ((a,update tt as v)#alist t))";
+      in Trie (value t) ((a,update tt as v) # alist t))";
 
 text{*\noindent
 The base case is obvious. In the recursive case the subtrie