src/Pure/System/ml_process.scala
author wenzelm
Tue, 08 Mar 2016 18:38:29 +0100
changeset 62560 498f6ff16804
parent 62557 a4ea3a222e0e
child 62563 2e352f63d15f
permissions -rw-r--r--
clarified initial ML;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     1
/*  Title:      Pure/System/ml_process.scala
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     2
    Author:     Makarius
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     3
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     4
The underlying ML process.
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     5
*/
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     6
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     7
package isabelle
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     8
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
     9
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    10
object ML_Process
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    11
{
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    12
  def apply(options: Options,
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    13
    heap: String = "",
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    14
    args: List[String] = Nil,
62556
c115e69f457f more abstract Session.start, without prover command-line;
wenzelm
parents: 62548
diff changeset
    15
    modes: List[String] = Nil,
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    16
    secure: Boolean = false,
62557
a4ea3a222e0e tuned signature;
wenzelm
parents: 62556
diff changeset
    17
    redirect: Boolean = false,
62556
c115e69f457f more abstract Session.start, without prover command-line;
wenzelm
parents: 62548
diff changeset
    18
    process_socket: String = ""): Bash.Process =
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    19
  {
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    20
    val load_heaps =
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    21
    {
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    22
      if (heap == "RAW_ML_SYSTEM") Nil
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    23
      else if (heap.iterator.contains('/')) {
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    24
        val heap_path = Path.explode(heap)
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    25
        if (!heap_path.is_file) error("Bad heap file: " + heap_path)
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    26
        List(heap_path)
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    27
      }
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    28
      else {
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    29
        val dirs = Isabelle_System.find_logics_dirs()
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    30
        val heap_name = if (heap == "") Isabelle_System.getenv_strict("ISABELLE_LOGIC") else heap
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    31
        dirs.map(_ + Path.basic(heap_name)).find(_.is_file) match {
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    32
          case Some(heap_path) => List(heap_path)
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    33
          case None =>
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    34
            error("Unknown logic " + quote(heap) + " -- no heap file found in:\n" +
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    35
              cat_lines(dirs.map(dir => "  " + dir.implode)))
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    36
        }
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    37
      }
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    38
    }
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    39
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    40
    val eval_heaps =
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    41
      load_heaps.map(load_heap =>
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    42
        "PolyML.SaveState.loadState " + ML_Syntax.print_string_raw(File.platform_path(load_heap)) +
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    43
        " handle exn => (TextIO.output (TextIO.stdErr, General.exnMessage exn ^ " +
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    44
        ML_Syntax.print_string_raw(": " + load_heap.toString + "\n") +
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    45
        "); OS.Process.exit OS.Process.failure)")
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    46
62560
498f6ff16804 clarified initial ML;
wenzelm
parents: 62557
diff changeset
    47
    val eval_initial =
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    48
      if (load_heaps.isEmpty) {
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    49
        List(
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    50
          if (Platform.is_windows)
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    51
            "fun exit 0 = OS.Process.exit OS.Process.success" +
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    52
            " | exit 1 = OS.Process.exit OS.Process.failure" +
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    53
            " | exit rc = OS.Process.exit (RunCall.unsafeCast (Word8.fromInt rc))"
62560
498f6ff16804 clarified initial ML;
wenzelm
parents: 62557
diff changeset
    54
          else
498f6ff16804 clarified initial ML;
wenzelm
parents: 62557
diff changeset
    55
            "fun exit rc = Posix.Process.exit (Word8.fromInt rc)",
498f6ff16804 clarified initial ML;
wenzelm
parents: 62557
diff changeset
    56
          "PolyML.Compiler.prompt1 := \"ML> \"",
498f6ff16804 clarified initial ML;
wenzelm
parents: 62557
diff changeset
    57
          "PolyML.Compiler.prompt2 := \"ML# \"",
62547
b33dea503665 clarified RAW_ML_SYSTEM;
wenzelm
parents: 62546
diff changeset
    58
          "PolyML.print_depth 10")
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    59
      }
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    60
      else Nil
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    61
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    62
    val eval_modes =
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    63
      if (modes.isEmpty) Nil
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    64
      else List("Print_Mode.add_modes " + ML_Syntax.print_list(ML_Syntax.print_string_raw _)(modes))
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    65
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    66
    // options
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    67
    val isabelle_process_options = Isabelle_System.tmp_file("options")
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    68
    File.write(isabelle_process_options, YXML.string_of_body(options.encode))
62545
8ebffdaf2ce2 Bash.process always uses a closed script instead of an open argument list, for extra robustness on Windows, where quoting is not well-defined;
wenzelm
parents: 62544
diff changeset
    69
    val env = Map("ISABELLE_PROCESS_OPTIONS" -> File.standard_path(isabelle_process_options))
62547
b33dea503665 clarified RAW_ML_SYSTEM;
wenzelm
parents: 62546
diff changeset
    70
    val eval_options = if (load_heaps.isEmpty) Nil else List("Options.load_default ()")
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    71
62556
c115e69f457f more abstract Session.start, without prover command-line;
wenzelm
parents: 62548
diff changeset
    72
    val eval_secure = if (secure) List("Secure.set_secure ()") else Nil
c115e69f457f more abstract Session.start, without prover command-line;
wenzelm
parents: 62548
diff changeset
    73
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    74
    val eval_process =
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    75
      if (process_socket == "") Nil
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    76
      else List("Isabelle_Process.init " + ML_Syntax.print_string_raw(process_socket))
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    77
62545
8ebffdaf2ce2 Bash.process always uses a closed script instead of an open argument list, for extra robustness on Windows, where quoting is not well-defined;
wenzelm
parents: 62544
diff changeset
    78
    // bash
8ebffdaf2ce2 Bash.process always uses a closed script instead of an open argument list, for extra robustness on Windows, where quoting is not well-defined;
wenzelm
parents: 62544
diff changeset
    79
    val bash_args =
8ebffdaf2ce2 Bash.process always uses a closed script instead of an open argument list, for extra robustness on Windows, where quoting is not well-defined;
wenzelm
parents: 62544
diff changeset
    80
      Word.explode(Isabelle_System.getenv("ML_OPTIONS")) :::
62560
498f6ff16804 clarified initial ML;
wenzelm
parents: 62557
diff changeset
    81
      (eval_heaps ::: eval_initial ::: eval_modes ::: eval_options ::: eval_secure ::: eval_process).
62545
8ebffdaf2ce2 Bash.process always uses a closed script instead of an open argument list, for extra robustness on Windows, where quoting is not well-defined;
wenzelm
parents: 62544
diff changeset
    82
        map(eval => List("--eval", eval)).flatten ::: args
62546
wenzelm
parents: 62545
diff changeset
    83
62557
a4ea3a222e0e tuned signature;
wenzelm
parents: 62556
diff changeset
    84
    Bash.process(env = env, redirect = redirect, script =
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    85
      """
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    86
        [ -z "$ISABELLE_TMP_PREFIX" ] && ISABELLE_TMP_PREFIX=/tmp/isabelle
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    87
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    88
        export ISABELLE_PID="$$"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    89
        export ISABELLE_TMP="$ISABELLE_TMP_PREFIX$ISABELLE_PID"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    90
        mkdir -p "$ISABELLE_TMP"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    91
        chmod $(umask -S) "$ISABELLE_TMP"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    92
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    93
        librarypath "$ML_HOME"
62548
f8ebb715e06d clarified treatment of DEL;
wenzelm
parents: 62547
diff changeset
    94
        "$ML_HOME/poly" -q -i """ + File.bash_args(bash_args) + """
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    95
        RC="$?"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    96
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    97
        rm -f "$ISABELLE_PROCESS_OPTIONS"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    98
        rmdir "$ISABELLE_TMP"
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
    99
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
   100
        exit "$RC"
62546
wenzelm
parents: 62545
diff changeset
   101
      """)
62544
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
   102
  }
efa178abe023 manage the underlying ML process in Scala;
wenzelm
parents:
diff changeset
   103
}