src/Pure/System/isabelle_process.scala
changeset 62634 aa3b47b32100
parent 62633 e57416b649d5
child 62668 360d3464919c
--- a/src/Pure/System/isabelle_process.scala	Tue Mar 15 23:59:39 2016 +0100
+++ b/src/Pure/System/isabelle_process.scala	Wed Mar 16 11:45:25 2016 +0100
@@ -11,7 +11,7 @@
 {
   def apply(
     options: Options,
-    heap: String = "",
+    logic: String = "",
     args: List[String] = Nil,
     modes: List[String] = Nil,
     secure: Boolean = false,
@@ -21,7 +21,7 @@
     val channel = System_Channel()
     val process =
       try {
-        ML_Process(options, heap = heap, args = args, modes = modes, secure = secure,
+        ML_Process(options, logic = logic, args = args, modes = modes, secure = secure,
           channel = Some(channel), store = store)
       }
       catch { case exn @ ERROR(_) => channel.accepted(); throw exn }