Trait/Object

virtufin.math

SymmetricMatrix

Related Docs: object SymmetricMatrix | package math

Permalink

trait SymmetricMatrix[V] extends Matrix[V]

Linear Supertypes
Known Subclasses
Type Hierarchy Learn more about scaladoc diagrams
Ordering
  1. Alphabetic
  2. By inheritance
Inherited
  1. SymmetricMatrix
  2. Matrix
  3. AnyRef
  4. Any
Implicitly
  1. by toRealMatrix
  2. by any2stringadd
  3. by StringFormat
  4. by Ensuring
  5. by ArrowAssoc
  1. Hide All
  2. Show all
Visibility
  1. Public
  2. All

Abstract Value Members

  1. abstract def apply(i: Int, j: Int): V

    Permalink
    Definition Classes
    SymmetricMatrixMatrix
  2. abstract def dimension: Int

    Permalink
  3. abstract def dimensions: (Int, Int)

    Permalink
    Definition Classes
    Matrix

Concrete 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 SymmetricMatrix[V] to any2stringadd[SymmetricMatrix[V]] performed by method any2stringadd in scala.Predef.
    Definition Classes
    any2stringadd
  4. def ->[B](y: B): (SymmetricMatrix[V], B)

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

    Permalink
    Definition Classes
    AnyRef → Any
  6. def add(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  7. def addToEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  8. final def asInstanceOf[T0]: T0

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

    Permalink
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  10. def copy(): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  11. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... ) @throws( ... )
  12. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... )
  13. def createMatrix(arg0: Int, arg1: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  14. def ensuring(cond: (SymmetricMatrix[V]) ⇒ Boolean, msg: ⇒ Any): SymmetricMatrix[V]

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

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

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

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

    Permalink
    Definition Classes
    AnyRef
  19. def equals(arg0: Any): Boolean

    Permalink
    Definition Classes
    AnyRef → Any
  20. def finalize(): Unit

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

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

    Permalink
    Definition Classes
    AnyRef → Any
  23. def getColumn(arg0: Int): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  24. def getColumnDimension(): Int

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    AnyMatrix
  25. def getColumnMatrix(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  26. def getColumnVector(arg0: Int): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  27. def getData(): Array[Array[Double]]

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  28. def getEntry(arg0: Int, arg1: Int): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  29. def getFrobeniusNorm(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  30. def getNorm(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  31. def getRow(arg0: Int): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  32. def getRowDimension(): Int

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    AnyMatrix
  33. def getRowMatrix(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  34. def getRowVector(arg0: Int): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  35. def getSubMatrix(arg0: Array[Int], arg1: Array[Int]): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... )
  36. def getSubMatrix(arg0: Int, arg1: Int, arg2: Int, arg3: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  37. def getTrace(): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  38. def hashCode(): Int

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

    Permalink
    Definition Classes
    Any
  40. def isSquare(): Boolean

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    AnyMatrix
  41. def multiply(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  42. def multiplyEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  43. final def ne(arg0: AnyRef): Boolean

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

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

    Permalink
    Definition Classes
    AnyRef
  46. def operate(arg0: RealVector): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  47. def operate(arg0: Array[Double]): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  48. def power(arg0: Int): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  49. def preMultiply(arg0: RealVector): RealVector

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  50. def preMultiply(arg0: Array[Double]): Array[Double]

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  51. def preMultiply(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  52. def scalarAdd(arg0: Double): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  53. def scalarMultiply(arg0: Double): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  54. def setColumn(arg0: Int, arg1: Array[Double]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  55. def setColumnMatrix(arg0: Int, arg1: RealMatrix): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  56. def setColumnVector(arg0: Int, arg1: RealVector): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  57. def setEntry(arg0: Int, arg1: Int, arg2: Double): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  58. def setRow(arg0: Int, arg1: Array[Double]): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  59. def setRowMatrix(arg0: Int, arg1: RealMatrix): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  60. def setRowVector(arg0: Int, arg1: RealVector): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  61. def setSubMatrix(arg0: Array[Array[Double]], arg1: Int, arg2: Int): Unit

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... ) @throws( ... ) @throws( ... )
  62. def subtract(arg0: RealMatrix): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... )
  63. final def synchronized[T0](arg0: ⇒ T0): T0

    Permalink
    Definition Classes
    AnyRef
  64. def toString(): String

    Permalink
    Definition Classes
    AnyRef → Any
  65. def transpose(): RealMatrix

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  66. final def wait(): Unit

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

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

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  69. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  70. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  71. def walkInColumnOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  72. def walkInColumnOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  73. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  74. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  75. def walkInOptimizedOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  76. def walkInOptimizedOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  77. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  78. 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 SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
    Annotations
    @throws( ... ) @throws( ... )
  79. def walkInRowOrder(arg0: RealMatrixPreservingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  80. def walkInRowOrder(arg0: RealMatrixChangingVisitor): Double

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to RealMatrix performed by method toRealMatrix in virtufin.math.Matrix. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    RealMatrix
  81. def [B](y: B): (SymmetricMatrix[V], B)

    Permalink
    Implicit information
    This member is added by an implicit conversion from SymmetricMatrix[V] to ArrowAssoc[SymmetricMatrix[V]] performed by method ArrowAssoc in scala.Predef. This conversion will take place only if V is Double (V =:= Double).
    Definition Classes
    ArrowAssoc

Inherited from Matrix[V]

Inherited from AnyRef

Inherited from Any

Inherited by implicit conversion toRealMatrix from SymmetricMatrix[V] to RealMatrix

Inherited by implicit conversion any2stringadd from SymmetricMatrix[V] to any2stringadd[SymmetricMatrix[V]]

Inherited by implicit conversion StringFormat from SymmetricMatrix[V] to StringFormat[SymmetricMatrix[V]]

Inherited by implicit conversion Ensuring from SymmetricMatrix[V] to Ensuring[SymmetricMatrix[V]]

Inherited by implicit conversion ArrowAssoc from SymmetricMatrix[V] to ArrowAssoc[SymmetricMatrix[V]]

Ungrouped