src/HOL/Enum.thy
changeset 58101 e7ebe5554281
parent 57922 dc78785427d0
child 58152 6fe60a9a5bad
--- a/src/HOL/Enum.thy	Sun Aug 31 09:10:41 2014 +0200
+++ b/src/HOL/Enum.thy	Sun Aug 31 09:10:42 2014 +0200
@@ -3,7 +3,7 @@
 header {* Finite types as explicit enumerations *}
 
 theory Enum
-imports Map
+imports Map Groups_List
 begin
 
 subsection {* Class @{text enum} *}