src/HOL/Word/Word.thy
changeset 67122 85b40f300fab
parent 67118 ccab07d1196c
child 67399 eab6ce8368fa
equal deleted inserted replaced
67121:116968454d70 67122:85b40f300fab
    12   Bool_List_Representation
    12   Bool_List_Representation
    13   Misc_Typedef
    13   Misc_Typedef
    14   Word_Miscellaneous
    14   Word_Miscellaneous
    15 begin
    15 begin
    16 
    16 
    17 text \<open>See \<^file>\<open>Examples/WordExamples.thy\<close> for examples.\<close>
    17 text \<open>See \<^file>\<open>WordExamples.thy\<close> for examples.\<close>
    18 
    18 
    19 subsection \<open>Type definition\<close>
    19 subsection \<open>Type definition\<close>
    20 
    20 
    21 typedef (overloaded) 'a word = "{(0::int) ..< 2 ^ len_of TYPE('a::len0)}"
    21 typedef (overloaded) 'a word = "{(0::int) ..< 2 ^ len_of TYPE('a::len0)}"
    22   morphisms uint Abs_word by auto
    22   morphisms uint Abs_word by auto