src/HOL/Word/Bits_Bit.thy
changeset 66453 cc19f7ca2ed6
parent 65363 5eb619751b14
child 67120 491fd7f0b5df
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Bit operations in $\cal Z_2$\<close>
     5 section \<open>Bit operations in $\cal Z_2$\<close>
     6 
     6 
     7 theory Bits_Bit
     7 theory Bits_Bit
     8 imports Bits "~~/src/HOL/Library/Bit"
     8 imports Bits "HOL-Library.Bit"
     9 begin
     9 begin
    10 
    10 
    11 instantiation bit :: bit
    11 instantiation bit :: bit
    12 begin
    12 begin
    13 
    13