src/HOL/Library/Code_Binary_Nat.thy
changeset 58881 b9556a055632
parent 55466 786edc984c98
child 60500 903bb1495239
equal deleted inserted replaced
58880:0baae4311a9f 58881:b9556a055632
     1 (*  Title:      HOL/Library/Code_Binary_Nat.thy
     1 (*  Title:      HOL/Library/Code_Binary_Nat.thy
     2     Author:     Florian Haftmann, TU Muenchen
     2     Author:     Florian Haftmann, TU Muenchen
     3 *)
     3 *)
     4 
     4 
     5 header {* Implementation of natural numbers as binary numerals *}
     5 section {* Implementation of natural numbers as binary numerals *}
     6 
     6 
     7 theory Code_Binary_Nat
     7 theory Code_Binary_Nat
     8 imports Code_Abstract_Nat
     8 imports Code_Abstract_Nat
     9 begin
     9 begin
    10 
    10