src/HOL/Option.thy
changeset 37880 3b9ca8d2c5fb
parent 36176 3fe7e97ccca8
child 38857 97775f3e8722
--- a/src/HOL/Option.thy	Mon Jul 19 11:55:42 2010 +0200
+++ b/src/HOL/Option.thy	Mon Jul 19 11:55:43 2010 +0200
@@ -114,7 +114,7 @@
   (SML "NONE" and "SOME")
   (OCaml "None" and "Some _")
   (Haskell "Nothing" and "Just")
-  (Scala "None" and "!Some((_))")
+  (Scala "!None" and "Some")
 
 code_instance option :: eq
   (Haskell -)