tuned signature: avoid aliases;
authorwenzelm
Sun, 22 Jan 2023 22:26:50 +0100
changeset 77044 a4380a2d6d2c
parent 77043 daf13aec9f04
child 77045 f51b0b54b20b
tuned signature: avoid aliases;
src/Pure/Admin/build_history.scala
src/Pure/Admin/other_isabelle.scala
--- a/src/Pure/Admin/build_history.scala	Sun Jan 22 22:19:28 2023 +0100
+++ b/src/Pure/Admin/build_history.scala	Sun Jan 22 22:26:50 2023 +0100
@@ -219,7 +219,7 @@
           tool <- List("ghc_setup", "ocaml_setup")
           if other_isabelle.getenv("ISABELLE_" + Word.uppercase(tool)) == "true" &&
             (other_isabelle.isabelle_home + Path.explode("lib/Tools/" + tool)).is_file
-        } other_isabelle(tool, echo = verbose)
+        } other_isabelle.bash("bin/isabelle " + tool, echo = verbose)
 
         Isabelle_System.rm_tree(isabelle_base_log)
       }
@@ -255,7 +255,7 @@
         Other_Isabelle(root, isabelle_identifier = isabelle_identifier,
           user_home = user_home, progress = build_out_progress)
       val build_result =
-        build_isabelle("build " + Bash.strings(build_args1 ::: afp_sessions),
+        build_isabelle.bash("bin/isabelle build " + Bash.strings(build_args1 ::: afp_sessions),
           redirect = true, echo = true, strict = false)
 
       val build_end = Date.now()
--- a/src/Pure/Admin/other_isabelle.scala	Sun Jan 22 22:19:28 2023 +0100
+++ b/src/Pure/Admin/other_isabelle.scala	Sun Jan 22 22:26:50 2023 +0100
@@ -44,23 +44,14 @@
       env = null, cwd = isabelle_home.file, redirect = redirect, echo = echo, strict = strict)
   }
 
-  def apply(
-    cmdline: String,
-    redirect: Boolean = false,
-    echo: Boolean = false,
-    strict: Boolean = true
-  ): Process_Result = {
-    bash("bin/isabelle " + cmdline, redirect = redirect, echo = echo, strict = strict)
-  }
-
   def resolve_components(echo: Boolean): Unit = {
-    other_isabelle(
-      "env ISABELLE_TOOLS=" + Bash.string(Isabelle_System.getenv("ISABELLE_TOOLS")) +
+    other_isabelle.bash(
+      "bin/isabelle env ISABELLE_TOOLS=" + Bash.string(Isabelle_System.getenv("ISABELLE_TOOLS")) +
       " isabelle components -a", redirect = true, echo = echo).check
   }
 
   def getenv(name: String): String =
-    other_isabelle("getenv -b " + Bash.string(name)).check.out
+    other_isabelle.bash("bin/isabelle getenv -b " + Bash.string(name)).check.out
 
   val isabelle_home_user: Path = Path.explode(getenv("ISABELLE_HOME_USER"))