Class

virtufin.math.Matrix

RealMatrixWrapper

Related Doc: package Matrix

Permalink

case class RealMatrixWrapper(m: RealMatrix) extends Matrix[Double] with Product with Serializable

Linear Supertypes
Type Hierarchy Learn more about scaladoc diagrams
Ordering
  1. Alphabetic
  2. By inheritance
Inherited
  1. RealMatrixWrapper
  2. Serializable
  3. Serializable
  4. Product
  5. Equals
  6. Matrix
  7. AnyRef
  8. Any
Implicitly
  1. by toRealMatrix
  2. by toRealMatrix
  3. by any2stringadd
  4. by StringFormat
  5. by Ensuring
  6. by ArrowAssoc
  1. Hide All
  2. Show all
Visibility
  1. Public
  2. All

Instance Constructors

  1. new RealMatrixWrapper(m: RealMatrix)

    Permalink

Value Members

  1. final def !=(arg0: Any): Boolean

    Permalink
    Definition Classes
    AnyRef → Any
  2. final def ##(): Int

    Permalink
    Definition Classes
    AnyRef → Any
  3. def +(other: String): String

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to any2stringadd[RealMatrixWrapper] performed by method any2stringadd in scala.Predef.
    Definition Classes
    any2stringadd
  4. def ->[B](y: B): (RealMatrixWrapper, B)

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to ArrowAssoc[RealMatrixWrapper] performed by method ArrowAssoc in scala.Predef.
    Definition Classes
    ArrowAssoc
    Annotations
    @inline()
  5. final def ==(arg0: Any): Boolean

    Permalink
    Definition Classes
    AnyRef → Any
  6. def apply(i: Int, j: Int): Double

    Permalink
    Definition Classes
    RealMatrixWrapperMatrix
  7. final def asInstanceOf[T0]: T0

    Permalink
    Definition Classes
    Any
  8. def clone(): AnyRef

    Permalink
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  9. def dimensions: (Int, Int)

    Permalink
    Definition Classes
    RealMatrixWrapperMatrix
  10. def ensuring(cond: (RealMatrixWrapper) ⇒ Boolean, msg: ⇒ Any): RealMatrixWrapper

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to Ensuring[RealMatrixWrapper] performed by method Ensuring in scala.Predef.
    Definition Classes
    Ensuring
  11. def ensuring(cond: (RealMatrixWrapper) ⇒ Boolean): RealMatrixWrapper

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to Ensuring[RealMatrixWrapper] performed by method Ensuring in scala.Predef.
    Definition Classes
    Ensuring
  12. def ensuring(cond: Boolean, msg: ⇒ Any): RealMatrixWrapper

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to Ensuring[RealMatrixWrapper] performed by method Ensuring in scala.Predef.
    Definition Classes
    Ensuring
  13. def ensuring(cond: Boolean): RealMatrixWrapper

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to Ensuring[RealMatrixWrapper] performed by method Ensuring in scala.Predef.
    Definition Classes
    Ensuring
  14. final def eq(arg0: AnyRef): Boolean

    Permalink
    Definition Classes
    AnyRef
  15. def finalize(): Unit

    Permalink
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( classOf[java.lang.Throwable] )
  16. def formatted(fmtstr: String): String

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to StringFormat[RealMatrixWrapper] performed by method StringFormat in scala.Predef.
    Definition Classes
    StringFormat
    Annotations
    @inline()
  17. final def getClass(): Class[_]

    Permalink
    Definition Classes
    AnyRef → Any
  18. final def isInstanceOf[T0]: Boolean

    Permalink
    Definition Classes
    Any
  19. val m: RealMatrix

    Permalink
  20. final def ne(arg0: AnyRef): Boolean

    Permalink
    Definition Classes
    AnyRef
  21. final def notify(): Unit

    Permalink
    Definition Classes
    AnyRef
  22. final def notifyAll(): Unit

    Permalink
    Definition Classes
    AnyRef
  23. final def synchronized[T0](arg0: ⇒ T0): T0

    Permalink
    Definition Classes
    AnyRef
  24. final def wait(): Unit

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  25. final def wait(arg0: Long, arg1: Int): Unit

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  26. final def wait(arg0: Long): Unit

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  27. def [B](y: B): (RealMatrixWrapper, B)

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to ArrowAssoc[RealMatrixWrapper] performed by method ArrowAssoc in scala.Predef.
    Definition Classes
    ArrowAssoc

Shadowed Implicit Value Members

  1. def add(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).add(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  2. def add(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).add(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  3. def addToEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).addToEntry(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  4. def addToEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).addToEntry(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  5. def copy(): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).copy()
    Definition Classes
    RealMatrix
  6. def copy(): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).copy()
    Definition Classes
    RealMatrix
  7. def copySubMatrix(arg0: Array[Int], arg1: Array[Int], arg2: Array[Array[Double]]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).copySubMatrix(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... ) @throws( ... )
  8. def copySubMatrix(arg0: Int, arg1: Int, arg2: Int, arg3: Int, arg4: Array[Array[Double]]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).copySubMatrix(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... )
  9. def copySubMatrix(arg0: Array[Int], arg1: Array[Int], arg2: Array[Array[Double]]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).copySubMatrix(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... ) @throws( ... )
  10. def copySubMatrix(arg0: Int, arg1: Int, arg2: Int, arg3: Int, arg4: Array[Array[Double]]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).copySubMatrix(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... )
  11. def createMatrix(arg0: Int, arg1: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).createMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  12. def createMatrix(arg0: Int, arg1: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).createMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  13. def getColumn(arg0: Int): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumn(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  14. def getColumn(arg0: Int): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumn(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  15. def getColumnDimension(): Int

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumnDimension()
    Definition Classes
    AnyMatrix
  16. def getColumnDimension(): Int

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumnDimension()
    Definition Classes
    AnyMatrix
  17. def getColumnMatrix(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumnMatrix(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  18. def getColumnMatrix(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumnMatrix(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  19. def getColumnVector(arg0: Int): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumnVector(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  20. def getColumnVector(arg0: Int): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getColumnVector(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  21. def getData(): Array[Array[Double]]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getData()
    Definition Classes
    RealMatrix
  22. def getData(): Array[Array[Double]]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getData()
    Definition Classes
    RealMatrix
  23. def getEntry(arg0: Int, arg1: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getEntry(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  24. def getEntry(arg0: Int, arg1: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getEntry(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  25. def getFrobeniusNorm(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getFrobeniusNorm()
    Definition Classes
    RealMatrix
  26. def getFrobeniusNorm(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getFrobeniusNorm()
    Definition Classes
    RealMatrix
  27. def getNorm(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getNorm()
    Definition Classes
    RealMatrix
  28. def getNorm(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getNorm()
    Definition Classes
    RealMatrix
  29. def getRow(arg0: Int): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRow(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  30. def getRow(arg0: Int): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRow(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  31. def getRowDimension(): Int

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRowDimension()
    Definition Classes
    AnyMatrix
  32. def getRowDimension(): Int

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRowDimension()
    Definition Classes
    AnyMatrix
  33. def getRowMatrix(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRowMatrix(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  34. def getRowMatrix(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRowMatrix(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  35. def getRowVector(arg0: Int): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRowVector(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  36. def getRowVector(arg0: Int): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getRowVector(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  37. def getSubMatrix(arg0: Array[Int], arg1: Array[Int]): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getSubMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... )
  38. def getSubMatrix(arg0: Int, arg1: Int, arg2: Int, arg3: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getSubMatrix(arg0, arg1, arg2, arg3)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  39. def getSubMatrix(arg0: Array[Int], arg1: Array[Int]): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getSubMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... )
  40. def getSubMatrix(arg0: Int, arg1: Int, arg2: Int, arg3: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getSubMatrix(arg0, arg1, arg2, arg3)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  41. def getTrace(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getTrace()
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  42. def getTrace(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).getTrace()
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  43. def isSquare(): Boolean

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).isSquare()
    Definition Classes
    AnyMatrix
  44. def isSquare(): Boolean

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).isSquare()
    Definition Classes
    AnyMatrix
  45. def multiply(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).multiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  46. def multiply(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).multiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  47. def multiplyEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).multiplyEntry(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  48. def multiplyEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).multiplyEntry(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  49. def operate(arg0: RealVector): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).operate(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  50. def operate(arg0: Array[Double]): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).operate(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  51. def operate(arg0: RealVector): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).operate(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  52. def operate(arg0: Array[Double]): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).operate(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  53. def power(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).power(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  54. def power(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).power(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  55. def preMultiply(arg0: RealVector): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).preMultiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  56. def preMultiply(arg0: Array[Double]): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).preMultiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  57. def preMultiply(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).preMultiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  58. def preMultiply(arg0: RealVector): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).preMultiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  59. def preMultiply(arg0: Array[Double]): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).preMultiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  60. def preMultiply(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).preMultiply(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  61. def scalarAdd(arg0: Double): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).scalarAdd(arg0)
    Definition Classes
    RealMatrix
  62. def scalarAdd(arg0: Double): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).scalarAdd(arg0)
    Definition Classes
    RealMatrix
  63. def scalarMultiply(arg0: Double): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).scalarMultiply(arg0)
    Definition Classes
    RealMatrix
  64. def scalarMultiply(arg0: Double): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).scalarMultiply(arg0)
    Definition Classes
    RealMatrix
  65. def setColumn(arg0: Int, arg1: Array[Double]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setColumn(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  66. def setColumn(arg0: Int, arg1: Array[Double]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setColumn(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  67. def setColumnMatrix(arg0: Int, arg1: RealMatrix): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setColumnMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  68. def setColumnMatrix(arg0: Int, arg1: RealMatrix): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setColumnMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  69. def setColumnVector(arg0: Int, arg1: RealVector): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setColumnVector(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  70. def setColumnVector(arg0: Int, arg1: RealVector): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setColumnVector(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  71. def setEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setEntry(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  72. def setEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setEntry(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  73. def setRow(arg0: Int, arg1: Array[Double]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setRow(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  74. def setRow(arg0: Int, arg1: Array[Double]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setRow(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  75. def setRowMatrix(arg0: Int, arg1: RealMatrix): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setRowMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  76. def setRowMatrix(arg0: Int, arg1: RealMatrix): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setRowMatrix(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  77. def setRowVector(arg0: Int, arg1: RealVector): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setRowVector(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  78. def setRowVector(arg0: Int, arg1: RealVector): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setRowVector(arg0, arg1)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  79. def setSubMatrix(arg0: Array[Array[Double]], arg1: Int, arg2: Int): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setSubMatrix(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... ) @throws( ... )
  80. def setSubMatrix(arg0: Array[Array[Double]], arg1: Int, arg2: Int): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).setSubMatrix(arg0, arg1, arg2)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... ) @throws( ... )
  81. def subtract(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).subtract(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  82. def subtract(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).subtract(arg0)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  83. def transpose(): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).transpose()
    Definition Classes
    RealMatrix
  84. def transpose(): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).transpose()
    Definition Classes
    RealMatrix
  85. def walkInColumnOrder(arg0: RealMatrixPreservingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  86. def walkInColumnOrder(arg0: RealMatrixChangingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  87. def walkInColumnOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0)
    Definition Classes
    RealMatrix
  88. def walkInColumnOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0)
    Definition Classes
    RealMatrix
  89. def walkInColumnOrder(arg0: RealMatrixPreservingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  90. def walkInColumnOrder(arg0: RealMatrixChangingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  91. def walkInColumnOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0)
    Definition Classes
    RealMatrix
  92. def walkInColumnOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInColumnOrder(arg0)
    Definition Classes
    RealMatrix
  93. def walkInOptimizedOrder(arg0: RealMatrixPreservingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  94. def walkInOptimizedOrder(arg0: RealMatrixChangingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  95. def walkInOptimizedOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0)
    Definition Classes
    RealMatrix
  96. def walkInOptimizedOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0)
    Definition Classes
    RealMatrix
  97. def walkInOptimizedOrder(arg0: RealMatrixPreservingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  98. def walkInOptimizedOrder(arg0: RealMatrixChangingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  99. def walkInOptimizedOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0)
    Definition Classes
    RealMatrix
  100. def walkInOptimizedOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInOptimizedOrder(arg0)
    Definition Classes
    RealMatrix
  101. def walkInRowOrder(arg0: RealMatrixPreservingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  102. def walkInRowOrder(arg0: RealMatrixChangingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  103. def walkInRowOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0)
    Definition Classes
    RealMatrix
  104. def walkInRowOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0)
    Definition Classes
    RealMatrix
  105. def walkInRowOrder(arg0: RealMatrixPreservingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  106. def walkInRowOrder(arg0: RealMatrixChangingVisitor, arg1: Int, arg2: Int, arg3: Int, arg4: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0, arg1, arg2, arg3, arg4)
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  107. def walkInRowOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0)
    Definition Classes
    RealMatrix
  108. def walkInRowOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from RealMatrixWrapper to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix.
    Shadowing
    This implicitly inherited member is ambiguous. One or more implicitly inherited members have similar signatures, so calling this member may produce an ambiguous implicit conversion compiler error.
    To access this member you can use a type ascription:
    (realMatrixWrapper: RealMatrix).walkInRowOrder(arg0)
    Definition Classes
    RealMatrix

Inherited from Serializable

Inherited from Serializable

Inherited from Product

Inherited from Equals

Inherited from Matrix[Double]

Inherited from AnyRef

Inherited from Any

Inherited by implicit conversion toRealMatrix from RealMatrixWrapper to RealMatrix

Inherited by implicit conversion toRealMatrix from RealMatrixWrapper to RealMatrix

Inherited by implicit conversion any2stringadd from RealMatrixWrapper to any2stringadd[RealMatrixWrapper]

Inherited by implicit conversion StringFormat from RealMatrixWrapper to StringFormat[RealMatrixWrapper]

Inherited by implicit conversion Ensuring from RealMatrixWrapper to Ensuring[RealMatrixWrapper]

Inherited by implicit conversion ArrowAssoc from RealMatrixWrapper to ArrowAssoc[RealMatrixWrapper]

Ungrouped