src/HOL/Library/Pretty_Int.thy
changeset 22949 997cef733bdd
parent 22803 5129e02f4df2
child 23859 fc44fa554ca8
equal deleted inserted replaced
22948:8752ca7f849a 22949:997cef733bdd
    17 
    17 
    18 code_type int
    18 code_type int
    19   (SML "IntInf.int")
    19   (SML "IntInf.int")
    20   (OCaml "Big'_int.big'_int")
    20   (OCaml "Big'_int.big'_int")
    21   (Haskell "Integer")
    21   (Haskell "Integer")
       
    22 
       
    23 code_instance int :: eq
       
    24   (Haskell -)
    22 
    25 
    23 setup {*
    26 setup {*
    24   fold (fn target => CodegenSerializer.add_pretty_numeral target
    27   fold (fn target => CodegenSerializer.add_pretty_numeral target
    25     (@{const_name number_of}, @{typ "int \<Rightarrow> int"})
    28     (@{const_name number_of}, @{typ "int \<Rightarrow> int"})
    26     @{const_name Numeral.B0} @{const_name Numeral.B1}
    29     @{const_name Numeral.B0} @{const_name Numeral.B1}