diff -r 6cbfe187a0f9 -r 6efff142bb54 src/HOL/Code_Numeral.thy --- a/src/HOL/Code_Numeral.thy Mon Jul 23 09:26:55 2012 +0200 +++ b/src/HOL/Code_Numeral.thy Mon Jul 23 09:28:03 2012 +0200 @@ -298,7 +298,7 @@ code_const "minus \ code_numeral \ code_numeral \ code_numeral" (SML "Int.max/ (0 : int,/ Int.-/ ((_),/ (_)))") (OCaml "Big'_int.max'_big'_int/ Big'_int.zero'_big'_int/ (Big'_int.sub'_big'_int/ _/ _)") - (Haskell "max/ (0 :: Integer)/ (_/ -/ _)") + (Haskell "Prelude.max/ (0 :: Integer)/ (_/ -/ _)") (Scala "!(_/ -/ _).max(0)") (Eval "Integer.max/ 0/ (_/ -/ _)")