src/HOL/Data_Structures/Tree23_Set.thy
changeset 67964 08cc5ab18c84
parent 67929 30486b96274d
child 67965 aaa31cd0caef
--- a/src/HOL/Data_Structures/Tree23_Set.thy	Sat Apr 07 22:09:57 2018 +0200
+++ b/src/HOL/Data_Structures/Tree23_Set.thy	Sun Apr 08 09:46:33 2018 +0200
@@ -6,7 +6,7 @@
 imports
   Tree23
   Cmp
-  Set_by_Ordered
+  Set_Interfaces
 begin
 
 fun isin :: "'a::linorder tree23 \<Rightarrow> 'a \<Rightarrow> bool" where