src/HOL/Int.thy
changeset 33364 2bd12592c5e8
parent 33336 5a989586d102
child 33523 96730ad673be
     1.1 --- a/src/HOL/Int.thy	Fri Oct 30 14:02:42 2009 +0100
     1.2 +++ b/src/HOL/Int.thy	Fri Oct 30 18:32:40 2009 +0100
     1.3 @@ -2246,13 +2246,13 @@
     1.4    by simp
     1.5  
     1.6  code_modulename SML
     1.7 -  Int Integer
     1.8 +  Int Arith
     1.9  
    1.10  code_modulename OCaml
    1.11 -  Int Integer
    1.12 +  Int Arith
    1.13  
    1.14  code_modulename Haskell
    1.15 -  Int Integer
    1.16 +  Int Arith
    1.17  
    1.18  types_code
    1.19    "int" ("int")