Packages

case class MPModel(solverLib: SolverLib = SolverLib.oJSolver) extends StrictLogging with Product with Serializable

Defines the mathematical programming model we are about to solve.

solverLib

a solver library (default is ojSolver)

Linear Supertypes
Serializable, Product, Equals, StrictLogging, AnyRef, Any
Ordering
  1. Alphabetic
  2. By Inheritance
Inherited
  1. MPModel
  2. Serializable
  3. Product
  4. Equals
  5. StrictLogging
  6. AnyRef
  7. Any
  1. Hide All
  2. Show All
Visibility
  1. Public
  2. Protected

Instance Constructors

  1. new MPModel(solverLib: SolverLib = SolverLib.oJSolver)

    solverLib

    a solver library (default is ojSolver)

Value Members

  1. final def !=(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  2. final def ##: Int
    Definition Classes
    AnyRef → Any
  3. final def ==(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  4. def add(constraint: Constraint): MPConstraint

    constraint

    a constraint to add

    returns

    an MPConstraint

    See also

    optimus.algebra.Constraint

  5. final def asInstanceOf[T0]: T0
    Definition Classes
    Any
  6. def checkConstraints(tol: Double = 10e-6): Boolean

    Check if all constraints in the model are satisfied by the given solution.

    Check if all constraints in the model are satisfied by the given solution.

    tol

    a tolerance threshold

    returns

    true if all constraints are satisfied, false otherwise

  7. def clone(): AnyRef
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.CloneNotSupportedException]) @native()
  8. val constraints: ArrayBuffer[MPConstraint]
    Attributes
    protected
  9. final def eq(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  10. def finalize(): Unit
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.Throwable])
  11. final def getClass(): Class[_ <: AnyRef]
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  12. def getStatus: SolutionStatus

    returns

    the status of the solution found for the model

  13. def getVarValue(idx: Int): Option[Double]

    idx

    the index of the variable

    returns

    the solution value for the variable

  14. final def isInstanceOf[T0]: Boolean
    Definition Classes
    Any
  15. val logger: Logger
    Attributes
    protected
    Definition Classes
    StrictLogging
  16. def maximize(expression: Expression): MPModel

    expression

    an expression to maximize

    returns

    the model

  17. def minimize(expression: Expression): MPModel

    expression

    an expression to minimize

    returns

    the model

  18. var minimize: Boolean
    Attributes
    protected
  19. final def ne(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  20. final def notify(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  21. final def notifyAll(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  22. var objective: Expression
    Attributes
    protected
  23. def objectiveValue: Double

    returns

    the objective value of the underlying solver

  24. def optimize(expression: Expression, minimize: Boolean): MPModel
    Attributes
    protected
  25. def productElementNames: Iterator[String]
    Definition Classes
    Product
  26. var reOptimize: Boolean
    Attributes
    protected
  27. def register(variable: MPVar): Int

    Register a variable to the model

    Register a variable to the model

    variable

    an MPVar to register

    returns

    the index of the variable

    See also

    optimus.optimization.model.MPVar

  28. def release(): Unit

    Release the memory of the underlying solver.

  29. var solution: HashMap[Int, Double]
    Attributes
    protected
  30. lazy val solver: MPSolver
    Attributes
    protected
  31. val solverLib: SolverLib
  32. def start(timeLimit: Int = Int.MaxValue, preSolve: PreSolve = DISABLED): Boolean

    Start the underlying solver.

    Start the underlying solver.

    timeLimit

    a time limit for the solver

    preSolve

    a pre solve strategy

    returns

    true if there is a solution, false otherwise

    See also

    optimus.optimization.enums.PreSolve

  33. final def synchronized[T0](arg0: => T0): T0
    Definition Classes
    AnyRef
  34. def variable(idx: Int): Try[MPVar]

    idx

    the index of the variable

    returns

    the MPVar on the given index

    See also

    optimus.optimization.model.MPVar

  35. val variables: ArrayBuffer[MPVar]
    Attributes
    protected
  36. final def wait(): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  37. final def wait(arg0: Long, arg1: Int): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  38. final def wait(arg0: Long): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException]) @native()

Inherited from Serializable

Inherited from Product

Inherited from Equals

Inherited from StrictLogging

Inherited from AnyRef

Inherited from Any

Ungrouped