tuned;
authorwenzelm
Tue, 05 Jan 2010 15:43:44 +0100
changeset 34263 2cb1530c2691
parent 34262 a6d2d9c07e46
child 34264 b5025782a4ed
tuned;
src/Pure/General/scan.scala
--- 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) =
       {