trait Start[F[_], PN] extends AnyRef
Type class for starting processes
- PN
Process type
- Alphabetic
- By Inheritance
- Start
- AnyRef
- Any
- Hide All
- Show All
- Public
- All
Type Members
- abstract type RunningProcessList <: HList
The RunningProcess instances returned by starting the process represented in a shapeless.HList
- abstract type RunningProcesses
The type returned by starting the processes holding one or more RunningProcess instances
Abstract Value Members
- abstract def apply(process: PN, dontStartOutput: Boolean = false, blocker: Blocker)(implicit concurrent: Concurrent[F], contextShift: ContextShift[F]): F[RunningProcesses]
Start the given process
Start the given process
The dontStartOutput option is used by the pipe construction as the output stream has to be connected to the second process' input channel first.
The input and error streams are always started.
- process
The process to be started
- dontStartOutput
Do no start the output redirection stream
- blocker
Execution context for the blocking stream IO
- contextShift
Context shifter to be used for the streams
- returns
Returns the RunningProcess instances of the started system processes
- abstract def toHList(process: PN, dontStartOutput: Boolean = false, blocker: Blocker)(implicit concurrent: Concurrent[F], contextShift: ContextShift[F]): F[RunningProcessList]
Start the given process
Start the given process
The dontStartOutput option is used by the pipe construction as the output stream has to be connected to the second process' input channel first.
The input and error streams are always started.
- process
The process to be started
- dontStartOutput
Do no start the output redirection stream
- blocker
Execution context for the blocking stream IO
- contextShift
Context shifter to be used for the streams
- returns
Returns the RunningProcess instances of the started system processes as a shapeless.HList
Concrete Value Members
- final def !=(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
- final def ##(): Int
- Definition Classes
- AnyRef → Any
- final def ==(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
- final def asInstanceOf[T0]: T0
- Definition Classes
- Any
- def clone(): AnyRef
- Attributes
- protected[java.lang]
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.CloneNotSupportedException]) @native()
- final def eq(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
- def equals(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef → Any
- def finalize(): Unit
- Attributes
- protected[java.lang]
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.Throwable])
- final def getClass(): Class[_ <: AnyRef]
- Definition Classes
- AnyRef → Any
- Annotations
- @native()
- def hashCode(): Int
- Definition Classes
- AnyRef → Any
- Annotations
- @native()
- final def isInstanceOf[T0]: Boolean
- Definition Classes
- Any
- final def ne(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
- final def notify(): Unit
- Definition Classes
- AnyRef
- Annotations
- @native()
- final def notifyAll(): Unit
- Definition Classes
- AnyRef
- Annotations
- @native()
- final def synchronized[T0](arg0: => T0): T0
- Definition Classes
- AnyRef
- def toString(): String
- Definition Classes
- AnyRef → Any
- final def wait(): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.InterruptedException])
- final def wait(arg0: Long, arg1: Int): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.InterruptedException])
- final def wait(arg0: Long): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.InterruptedException]) @native()