src/HOL/Library/Executable_Set.thy
changeset 33186 607b702feace
parent 32881 13b153243ed4
child 34022 bb37c95f0b8e
--- a/src/HOL/Library/Executable_Set.thy	Mon Oct 26 10:51:41 2009 +0100
+++ b/src/HOL/Library/Executable_Set.thy	Mon Oct 26 10:51:42 2009 +0100
@@ -5,7 +5,7 @@
 header {* Implementation of finite sets by lists *}
 
 theory Executable_Set
-imports Main Fset
+imports Main Fset SML_Quickcheck
 begin
 
 subsection {* Preprocessor setup *}