src/HOL/Product_Type.thy
changeset 34900 9b12b0824bfe
parent 34886 873c31d9f10d
child 35115 446c5063e4fd
--- a/src/HOL/Product_Type.thy	Thu Jan 14 17:47:39 2010 +0100
+++ b/src/HOL/Product_Type.thy	Thu Jan 14 17:47:39 2010 +0100
@@ -1000,7 +1000,7 @@
   (SML infix 2 "*")
   (OCaml infix 2 "*")
   (Haskell "!((_),/ (_))")
-  (Scala "!((_),/ (_))")
+  (Scala "((_),/ (_))")
 
 code_instance * :: eq
   (Haskell -)