doc-src/TutorialI/Trie/Trie.thy
changeset 16417 9bc16273c2d4
parent 15905 0a4cc9b113c7
child 17555 23c4a349feff
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     1 (*<*)
     1 (*<*)
     2 theory Trie = Main:;
     2 theory Trie imports Main begin;
     3 (*>*)
     3 (*>*)
     4 text{*
     4 text{*
     5 To minimize running time, each node of a trie should contain an array that maps
     5 To minimize running time, each node of a trie should contain an array that maps
     6 letters to subtries. We have chosen a
     6 letters to subtries. We have chosen a
     7 representation where the subtries are held in an association list, i.e.\ a
     7 representation where the subtries are held in an association list, i.e.\ a