src/HOL/Code_Numeral.thy
changeset 49446 6efff142bb54
parent 48116 30a1692557b0
child 50849 b27bbb021df1
     1.1 --- a/src/HOL/Code_Numeral.thy	Mon Jul 23 09:26:55 2012 +0200
     1.2 +++ b/src/HOL/Code_Numeral.thy	Mon Jul 23 09:28:03 2012 +0200
     1.3 @@ -298,7 +298,7 @@
     1.4  code_const "minus \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
     1.5    (SML "Int.max/ (0 : int,/ Int.-/ ((_),/ (_)))")
     1.6    (OCaml "Big'_int.max'_big'_int/ Big'_int.zero'_big'_int/ (Big'_int.sub'_big'_int/ _/ _)")
     1.7 -  (Haskell "max/ (0 :: Integer)/ (_/ -/ _)")
     1.8 +  (Haskell "Prelude.max/ (0 :: Integer)/ (_/ -/ _)")
     1.9    (Scala "!(_/ -/ _).max(0)")
    1.10    (Eval "Integer.max/ 0/ (_/ -/ _)")
    1.11