src/HOL/Word/Word.thy
changeset 53062 3af1a6020014
parent 51717 9e7d1c139569
child 53080 d815e25ead03
--- a/src/HOL/Word/Word.thy	Sun Aug 18 13:58:33 2013 +0200
+++ b/src/HOL/Word/Word.thy	Sun Aug 18 15:29:50 2013 +0200
@@ -7,9 +7,10 @@
 theory Word
 imports
   Type_Length
-  Misc_Typedef
   "~~/src/HOL/Library/Boolean_Algebra"
   Bool_List_Representation
+  Misc_Typedef
+  Word_Miscellaneous
 begin
 
 text {* see @{text "Examples/WordExamples.thy"} for examples *}