src/HOL/Code_Numeral.thy
changeset 66836 4eb431c3f974
parent 66817 0b12755ccbb2
child 66838 17989f6bc7b2
equal deleted inserted replaced
66835:ecc99a5a1ab8 66836:4eb431c3f974
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Numeric types for code generation onto target language numerals only\<close>
     5 section \<open>Numeric types for code generation onto target language numerals only\<close>
     6 
     6 
     7 theory Code_Numeral
     7 theory Code_Numeral
     8 imports Nat_Transfer Divides Lifting
     8 imports Divides Lifting
     9 begin
     9 begin
    10 
    10 
    11 subsection \<open>Type of target language integers\<close>
    11 subsection \<open>Type of target language integers\<close>
    12 
    12 
    13 typedef integer = "UNIV :: int set"
    13 typedef integer = "UNIV :: int set"