src/Pure/System/isabelle_process.scala
author wenzelm
Sat, 13 Feb 2016 20:41:56 +0100
changeset 62296 b04a5ddd6121
parent 60991 2fc5a44346b5
child 62299 9e95a4afb8c3
permissions -rw-r--r--
clarified bash process -- similar to ML version;

/*  Title:      Pure/System/isabelle_process.scala
    Author:     Makarius

Isabelle process wrapper.
*/

package isabelle


object Isabelle_Process
{
  def apply(
    receiver: Prover.Message => Unit = Console.println(_),
    prover_args: String = ""): Isabelle_Process =
  {
    val system_channel = System_Channel()
    val system_process =
      try {
        val script =
          "\"$ISABELLE_PROCESS\" " + system_channel.prover_options +
            (if (prover_args == "") "" else " " + prover_args)
        val process = Bash.process(null, null, false, "-c", script)
        process.stdin.close
        process
      }
      catch { case exn @ ERROR(_) => system_channel.accepted(); throw exn }

    new Isabelle_Process(receiver, system_channel, system_process)
  }
}

class Isabelle_Process private(
    receiver: Prover.Message => Unit,
    system_channel: System_Channel,
    system_process: Prover.System_Process)
  extends Prover(receiver, system_channel, system_process)
  {
    def encode(s: String): String = Symbol.encode(s)
    def decode(s: String): String = Symbol.decode(s)
  }