src/Pure/Tools/build_process.scala
changeset 78178 a177f71dc79f
parent 78175 a081ad6c3c4b
child 78179 a49ad8d183af
equal deleted inserted replaced
78177:ea7a3cc64df5 78178:a177f71dc79f
    16 object Build_Process {
    16 object Build_Process {
    17   /** static context **/
    17   /** static context **/
    18 
    18 
    19   object Context {
    19   object Context {
    20     def apply(
    20     def apply(
    21       store: Sessions.Store,
    21       store: Store,
    22       build_deps: Sessions.Deps,
    22       build_deps: Sessions.Deps,
    23       progress: Progress = new Progress,
    23       progress: Progress = new Progress,
    24       ml_platform: String = Isabelle_System.getenv("ML_PLATFORM"),
    24       ml_platform: String = Isabelle_System.getenv("ML_PLATFORM"),
    25       hostname: String = Isabelle_System.hostname(),
    25       hostname: String = Isabelle_System.hostname(),
    26       numa_shuffling: Boolean = false,
    26       numa_shuffling: Boolean = false,
    87         no_build = no_build, session_setup, build_uuid = build_uuid, master = master)
    87         no_build = no_build, session_setup, build_uuid = build_uuid, master = master)
    88     }
    88     }
    89   }
    89   }
    90 
    90 
    91   final class Context private(
    91   final class Context private(
    92     val store: Sessions.Store,
    92     val store: Store,
    93     val build_deps: Sessions.Deps,
    93     val build_deps: Sessions.Deps,
    94     val sessions: State.Sessions,
    94     val sessions: State.Sessions,
    95     val ordering: Ordering[String],
    95     val ordering: Ordering[String],
    96     val ml_platform: String,
    96     val ml_platform: String,
    97     val hostname: String,
    97     val hostname: String,
   794   protected final val build_progress: Progress
   794   protected final val build_progress: Progress
   795 )
   795 )
   796 extends AutoCloseable {
   796 extends AutoCloseable {
   797   /* context */
   797   /* context */
   798 
   798 
   799   protected final val store: Sessions.Store = build_context.store
   799   protected final val store: Store = build_context.store
   800   protected final val build_options: Options = store.options
   800   protected final val build_options: Options = store.options
   801   protected final val build_deps: Sessions.Deps = build_context.build_deps
   801   protected final val build_deps: Sessions.Deps = build_context.build_deps
   802   protected final val hostname: String = build_context.hostname
   802   protected final val hostname: String = build_context.hostname
   803   protected final val build_uuid: String = build_context.build_uuid
   803   protected final val build_uuid: String = build_context.build_uuid
   804 
   804