src/HOL/Code_Numeral.thy
changeset 34944 970e1466028d
parent 34917 51829fe604a7
child 35028 108662d50512
equal deleted inserted replaced
34943:e97b22500a5c 34944:970e1466028d
   294 code_instance code_numeral :: eq
   294 code_instance code_numeral :: eq
   295   (Haskell -)
   295   (Haskell -)
   296 
   296 
   297 setup {*
   297 setup {*
   298   fold (Numeral.add_code @{const_name number_code_numeral_inst.number_of_code_numeral}
   298   fold (Numeral.add_code @{const_name number_code_numeral_inst.number_of_code_numeral}
   299     false false Code_Printer.str) ["SML", "Haskell"]
   299     false Code_Printer.literal_naive_numeral) ["SML", "Haskell"]
   300   #> Numeral.add_code @{const_name number_code_numeral_inst.number_of_code_numeral}
   300   #> Numeral.add_code @{const_name number_code_numeral_inst.number_of_code_numeral}
   301     false true Code_Printer.str "OCaml"
   301     false Code_Printer.literal_numeral "OCaml"
   302   #> Numeral.add_code @{const_name number_code_numeral_inst.number_of_code_numeral}
   302   #> Numeral.add_code @{const_name number_code_numeral_inst.number_of_code_numeral}
   303     false false Code_Printer.str "Scala"
   303     false Code_Printer.literal_naive_numeral "Scala"
   304 *}
   304 *}
   305 
   305 
   306 code_reserved SML Int int
   306 code_reserved SML Int int
   307 code_reserved OCaml Big_int
       
   308 code_reserved Scala Int
   307 code_reserved Scala Int
   309 
   308 
   310 code_const "op + \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
   309 code_const "op + \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
   311   (SML "Int.+/ ((_),/ (_))")
   310   (SML "Int.+/ ((_),/ (_))")
   312   (OCaml "Big'_int.add'_big'_int")
   311   (OCaml "Big'_int.add'_big'_int")