src/HOL/Library/Code_Target_Nat.thy
changeset 52435 6646bb548c6b
parent 51143 0a2371e7ced3
child 53027 1774d569b604
equal deleted inserted replaced
52434:cbb94074682b 52435:6646bb548c6b
   121 
   121 
   122 lemma [code abstract]:
   122 lemma [code abstract]:
   123   "integer_of_nat (nat k) = max 0 (integer_of_int k)"
   123   "integer_of_nat (nat k) = max 0 (integer_of_int k)"
   124   by transfer auto
   124   by transfer auto
   125 
   125 
   126 code_modulename SML
   126 code_identifier
   127   Code_Target_Nat Arith
   127   code_module Code_Target_Nat \<rightharpoonup>
   128 
   128     (SML) Arith and (OCaml) Arith and (Haskell) Arith
   129 code_modulename OCaml
       
   130   Code_Target_Nat Arith
       
   131 
       
   132 code_modulename Haskell
       
   133   Code_Target_Nat Arith
       
   134 
   129 
   135 end
   130 end
   136 
   131