src/HOL/Word/Word.thy
changeset 66453 cc19f7ca2ed6
parent 65363 5eb619751b14
child 66808 1907167b6038
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     4 
     4 
     5 section \<open>A type of finite bit strings\<close>
     5 section \<open>A type of finite bit strings\<close>
     6 
     6 
     7 theory Word
     7 theory Word
     8 imports
     8 imports
     9   "~~/src/HOL/Library/Type_Length"
     9   "HOL-Library.Type_Length"
    10   "~~/src/HOL/Library/Boolean_Algebra"
    10   "HOL-Library.Boolean_Algebra"
    11   Bits_Bit
    11   Bits_Bit
    12   Bool_List_Representation
    12   Bool_List_Representation
    13   Misc_Typedef
    13   Misc_Typedef
    14   Word_Miscellaneous
    14   Word_Miscellaneous
    15 begin
    15 begin