src/HOL/Library/RBT.thy
changeset 53013 3fbcfa911863
parent 51375 d9e62d9c98de
child 55414 eab03e9cee8a
--- a/src/HOL/Library/RBT.thy	Tue Aug 13 15:59:22 2013 +0200
+++ b/src/HOL/Library/RBT.thy	Tue Aug 13 15:59:22 2013 +0200
@@ -5,7 +5,7 @@
 header {* Abstract type of RBT trees *}
 
 theory RBT 
-imports Main RBT_Impl Quotient_List
+imports Main RBT_Impl
 begin
 
 subsection {* Type definition *}