src/Pure/System/isabelle_platform.scala
changeset 75393 87ebf5a50283
parent 73716 00ef0f401a29
child 77328 f30e050d4ac6
--- a/src/Pure/System/isabelle_platform.scala	Fri Apr 01 11:51:42 2022 +0200
+++ b/src/Pure/System/isabelle_platform.scala	Fri Apr 01 17:06:10 2022 +0200
@@ -7,8 +7,7 @@
 package isabelle
 
 
-object Isabelle_Platform
-{
+object Isabelle_Platform {
   val settings: List[String] =
     List(
       "ISABELLE_PLATFORM_FAMILY",
@@ -17,8 +16,7 @@
       "ISABELLE_WINDOWS_PLATFORM64",
       "ISABELLE_APPLE_PLATFORM64")
 
-  def apply(ssh: Option[SSH.Session] = None): Isabelle_Platform =
-  {
+  def apply(ssh: Option[SSH.Session] = None): Isabelle_Platform = {
     ssh match {
       case None =>
         new Isabelle_Platform(settings.map(a => (a, Isabelle_System.getenv(a))))
@@ -36,8 +34,7 @@
   lazy val self: Isabelle_Platform = apply()
 }
 
-class Isabelle_Platform private(val settings: List[(String, String)])
-{
+class Isabelle_Platform private(val settings: List[(String, String)]) {
   private def get(name: String): String =
     settings.collectFirst({ case (a, b) if a == name => b }).
       getOrElse(error("Bad platform settings variable: " + quote(name)))