src/HOL/Library/Code_Integer.thy
changeset 38185 844977c7abeb
parent 34931 970e1466028d
child 38195 9728342bcd56
equal deleted inserted replaced
38184:be3c0df7bb90 38185:844977c7abeb
   110   (Scala infixl 4 "<=")
   110   (Scala infixl 4 "<=")
   111 
   111 
   112 code_const Code_Numeral.int_of
   112 code_const Code_Numeral.int_of
   113   (SML "IntInf.fromInt")
   113   (SML "IntInf.fromInt")
   114   (OCaml "_")
   114   (OCaml "_")
   115   (Haskell "toEnum")
   115   (Haskell "_")
   116   (Scala "!BigInt((_))")
   116   (Scala "!BigInt((_))")
   117 
   117 
   118 text {* Evaluation *}
   118 text {* Evaluation *}
   119 
   119 
   120 code_const "Code_Evaluation.term_of \<Colon> int \<Rightarrow> term"
   120 code_const "Code_Evaluation.term_of \<Colon> int \<Rightarrow> term"