src/HOL/Code_Numeral.thy
changeset 46567 4a8743618257
parent 45692 a92f65e174cf
child 46899 9f113cdf3d66
equal deleted inserted replaced
46566:bbd2c7ffc02c 46567:4a8743618257
    12 *}
    12 *}
    13 
    13 
    14 subsection {* Datatype of target language numerals *}
    14 subsection {* Datatype of target language numerals *}
    15 
    15 
    16 typedef (open) code_numeral = "UNIV \<Colon> nat set"
    16 typedef (open) code_numeral = "UNIV \<Colon> nat set"
    17   morphisms nat_of of_nat by rule
    17   morphisms nat_of of_nat ..
    18 
    18 
    19 lemma of_nat_nat_of [simp]:
    19 lemma of_nat_nat_of [simp]:
    20   "of_nat (nat_of k) = k"
    20   "of_nat (nat_of k) = k"
    21   by (rule nat_of_inverse)
    21   by (rule nat_of_inverse)
    22 
    22