src/Pure/General/scan.scala
changeset 34263 2cb1530c2691
parent 34189 10c5871ec684
child 34267 92810c85262e
--- a/src/Pure/General/scan.scala	Tue Jan 05 13:45:17 2010 +0100
+++ b/src/Pure/General/scan.scala	Tue Jan 05 15:43:44 2010 +0100
@@ -220,8 +220,8 @@
       val comment_text =
         rep(many1(sym => sym != "*" && sym != "(" && Symbol.is_closed(sym)) |
           """\*(?!\))|\((?!\*)""".r)
-      val comment_open = "(*" ~ comment_text ^^ (_ => ())
-      val comment_close = comment_text ~ "*)" ^^ (_ => ())
+      val comment_open = "(*" ~ comment_text ^^^ ()
+      val comment_close = comment_text ~ "*)" ^^^ ()
 
       def apply(in: Input) =
       {