src/Pure/Admin/build_log.scala
changeset 73715 bf51c23f3f99
parent 73713 d95d34efbe6f
child 74782 0a87ea7eb76f
--- a/src/Pure/Admin/build_log.scala	Mon May 17 14:07:13 2021 +0200
+++ b/src/Pure/Admin/build_log.scala	Mon May 17 14:07:51 2021 +0200
@@ -63,7 +63,7 @@
         for { (a, b) <- Properties.Eq.unapply(s) }
         yield (a, Library.perhaps_unquote(b))
       def getenv(a: String): String =
-        Properties.Eq(a -> quote(Isabelle_System.getenv(a)))
+        Properties.Eq(a, quote(Isabelle_System.getenv(a)))
     }
 
     def show(): String =
@@ -226,8 +226,8 @@
 
     /* settings */
 
-    def get_setting(a: String): Option[Settings.Entry] =
-      lines.collectFirst({ case Settings.Entry(entry) if entry._1 == a => entry })
+    def get_setting(name: String): Option[Settings.Entry] =
+      lines.collectFirst({ case Settings.Entry(a, b) if a == name => a -> b })
 
     def get_all_settings: Settings.T =
       for { c <- Settings.all_settings; entry <- get_setting(c.name) }