src/Pure/Admin/build_log.scala
changeset 73712 3eba8d4b624b
parent 73344 f5c147654661
child 73713 d95d34efbe6f
--- a/src/Pure/Admin/build_log.scala	Mon May 17 13:37:47 2021 +0200
+++ b/src/Pure/Admin/build_log.scala	Mon May 17 13:40:01 2021 +0200
@@ -60,14 +60,9 @@
     object Entry
     {
       def unapply(s: String): Option[Entry] =
-        s.indexOf('=') match {
-          case -1 => None
-          case i =>
-            val a = s.substring(0, i)
-            val b = Library.perhaps_unquote(s.substring(i + 1))
-            Some((a, b))
-        }
-      def apply(a: String, b: String): String = a + "=" + quote(b)
+        for { (a, b) <- Properties.Eq.unapply(s) }
+        yield (a, Library.perhaps_unquote(b))
+      def apply(a: String, b: String): String = Properties.Eq(a -> quote(b))
       def getenv(a: String): String = apply(a, Isabelle_System.getenv(a))
     }