src/HOL/Data_Structures/Tree234_Set.thy
changeset 62130 90a3016a6c12
parent 61709 47f7263870a0
child 63411 e051eea34990
equal deleted inserted replaced
62129:72d19e588e97 62130:90a3016a6c12
     1 (* Author: Tobias Nipkow *)
     1 (* Author: Tobias Nipkow *)
     2 
     2 
     3 section \<open>A 2-3-4 Tree Implementation of Sets\<close>
     3 section \<open>2-3-4 Tree Implementation of Sets\<close>
     4 
     4 
     5 theory Tree234_Set
     5 theory Tree234_Set
     6 imports
     6 imports
     7   Tree234
     7   Tree234
     8   Cmp
     8   Cmp