src/HOL/Data_Structures/Tree234_Set.thy
changeset 67964 08cc5ab18c84
parent 67929 30486b96274d
child 67965 aaa31cd0caef
--- a/src/HOL/Data_Structures/Tree234_Set.thy	Sat Apr 07 22:09:57 2018 +0200
+++ b/src/HOL/Data_Structures/Tree234_Set.thy	Sun Apr 08 09:46:33 2018 +0200
@@ -6,7 +6,7 @@
 imports
   Tree234
   Cmp
-  "../Data_Structures/Set_by_Ordered"
+  "Set_Interfaces"
 begin
 
 subsection \<open>Set operations on 2-3-4 trees\<close>