trait TensorLike[K, V, +This <: Tensor[K, V]] extends QuasiTensor[K, V] with NumericOps[This]
- Alphabetic
- By Inheritance
- TensorLike
- NumericOps
- ImmutableNumericOps
- QuasiTensor
- AnyRef
- Any
- Hide All
- Show All
- Public
- All
Abstract Value Members
-
abstract
def
activeIterator: Iterator[(K, V)]
- Definition Classes
- QuasiTensor
-
abstract
def
activeKeysIterator: Iterator[K]
- Definition Classes
- QuasiTensor
- abstract def activeSize: Int
-
abstract
def
activeValuesIterator: Iterator[V]
- Definition Classes
- QuasiTensor
-
abstract
def
apply(i: K): V
- Definition Classes
- TensorLike → QuasiTensor
-
abstract
def
iterator: Iterator[(K, V)]
- Definition Classes
- QuasiTensor
-
abstract
def
keySet: Set[K]
- Definition Classes
- QuasiTensor
-
abstract
def
keysIterator: Iterator[K]
- Definition Classes
- QuasiTensor
-
abstract
def
repr: This
- Definition Classes
- ImmutableNumericOps
- abstract def size: Int
-
abstract
def
update(i: K, v: V): Unit
- Definition Classes
- TensorLike → QuasiTensor
-
abstract
def
valuesIterator: Iterator[V]
- Definition Classes
- QuasiTensor
Concrete Value Members
-
final
def
!=(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
-
final
def
##(): Int
- Definition Classes
- AnyRef → Any
-
final
def
%[TT >: This, B, That](b: B)(implicit op: operators.OpMod.Impl2[TT, B, That]): That
Alias for :%(b) when b is a scalar.
Alias for :%(b) when b is a scalar.
- Definition Classes
- ImmutableNumericOps
-
final
def
%:%[TT >: This, B, That](b: B)(implicit op: operators.OpMod.Impl2[TT, B, That]): That
Element-wise modulo of this and b.
Element-wise modulo of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
%=[TT >: This, B](b: B)(implicit op: operators.OpMod.InPlaceImpl2[TT, B]): This
Alias for :%=(b) when b is a scalar.
Alias for :%=(b) when b is a scalar.
- Definition Classes
- NumericOps
-
final
def
&[TT >: This, B, That](b: B)(implicit op: operators.OpAnd.Impl2[TT, B, That]): That
Alias for :&&(b) for all b.
Alias for :&&(b) for all b.
- Definition Classes
- ImmutableNumericOps
-
final
def
&:&[TT >: This, B, That](b: B)(implicit op: operators.OpAnd.Impl2[TT, B, That]): That
Element-wise logical "and" operator -- returns true if corresponding elements are non-zero.
Element-wise logical "and" operator -- returns true if corresponding elements are non-zero.
- Definition Classes
- ImmutableNumericOps
-
final
def
&=[TT >: This, B](b: B)(implicit op: operators.OpAnd.InPlaceImpl2[TT, B]): This
Mutates this by element-wise and of this and b.
Mutates this by element-wise and of this and b.
- Definition Classes
- NumericOps
-
final
def
*[TT >: This, B, That](b: B)(implicit op: operators.OpMulMatrix.Impl2[TT, B, That]): That
Matrix multiplication (and scalar multiplication that follows standard order of operations)
Matrix multiplication (and scalar multiplication that follows standard order of operations)
- Definition Classes
- ImmutableNumericOps
-
final
def
*:*[TT >: This, B, That](b: B)(implicit op: operators.OpMulScalar.Impl2[TT, B, That]): That
Element-wise product of this and b.
Element-wise product of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
*=[TT >: This, B](b: B)(implicit op: operators.OpMulScalar.InPlaceImpl2[TT, B]): This
Alias for :*=(b) when b is a scalar.
Alias for :*=(b) when b is a scalar.
- Definition Classes
- NumericOps
-
final
def
+[TT >: This, B, C, That](b: B)(implicit op: operators.OpAdd.Impl2[TT, B, That]): That
Alias for :+(b) for all b.
Alias for :+(b) for all b.
- Definition Classes
- NumericOps
-
final
def
+:+[TT >: This, B, That](b: B)(implicit op: operators.OpAdd.Impl2[TT, B, That]): That
Element-wise sum of this and b.
Element-wise sum of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
+=[TT >: This, B](b: B)(implicit op: operators.OpAdd.InPlaceImpl2[TT, B]): This
Alias for :+=(b) for all b.
Alias for :+=(b) for all b.
- Definition Classes
- NumericOps
-
final
def
-[TT >: This, B, That](b: B)(implicit op: operators.OpSub.Impl2[TT, B, That]): That
Alias for :-(b) for all b.
Alias for :-(b) for all b.
- Definition Classes
- ImmutableNumericOps
-
final
def
-:-[TT >: This, B, That](b: B)(implicit op: operators.OpSub.Impl2[TT, B, That]): That
Element-wise difference of this and b.
Element-wise difference of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
-=[TT >: This, B](b: B)(implicit op: operators.OpSub.InPlaceImpl2[TT, B]): This
Alias for :-=(b) for all b.
Alias for :-=(b) for all b.
- Definition Classes
- NumericOps
-
final
def
/[TT >: This, B, That](b: B)(implicit op: operators.OpDiv.Impl2[TT, B, That]): That
Alias for :/(b) when b is a scalar.
Alias for :/(b) when b is a scalar.
- Definition Classes
- ImmutableNumericOps
-
final
def
/:/[TT >: This, B, That](b: B)(implicit op: operators.OpDiv.Impl2[TT, B, That]): That
Element-wise quotient of this and b.
Element-wise quotient of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
/=[TT >: This, B](b: B)(implicit op: operators.OpDiv.InPlaceImpl2[TT, B]): This
Alias for :/=(b) when b is a scalar.
Alias for :/=(b) when b is a scalar.
- Definition Classes
- NumericOps
-
final
def
:!=[TT >: This, B, That](b: B)(implicit op: operators.OpNe.Impl2[TT, B, That]): That
Element-wise inequality comparator of this and b.
Element-wise inequality comparator of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
:%=[TT >: This, B](b: B)(implicit op: operators.OpMod.InPlaceImpl2[TT, B]): This
Mutates this by element-wise modulo of b into this.
Mutates this by element-wise modulo of b into this.
- Definition Classes
- NumericOps
-
final
def
:&=[TT >: This, B](b: B)(implicit op: operators.OpAnd.InPlaceImpl2[TT, B]): This
Mutates this by element-wise and of this and b.
Mutates this by element-wise and of this and b.
- Definition Classes
- NumericOps
-
final
def
:*=[TT >: This, B](b: B)(implicit op: operators.OpMulScalar.InPlaceImpl2[TT, B]): This
Mutates this by element-wise multiplication of b into this.
Mutates this by element-wise multiplication of b into this.
- Definition Classes
- NumericOps
-
final
def
:+=[TT >: This, B](b: B)(implicit op: operators.OpAdd.InPlaceImpl2[TT, B]): This
Mutates this by element-wise addition of b into this.
Mutates this by element-wise addition of b into this.
- Definition Classes
- NumericOps
-
final
def
:-=[TT >: This, B](b: B)(implicit op: operators.OpSub.InPlaceImpl2[TT, B]): This
Mutates this by element-wise subtraction of b from this
Mutates this by element-wise subtraction of b from this
- Definition Classes
- NumericOps
-
final
def
:/=[TT >: This, B](b: B)(implicit op: operators.OpDiv.InPlaceImpl2[TT, B]): This
Mutates this by element-wise division of b into this
Mutates this by element-wise division of b into this
- Definition Classes
- NumericOps
-
final
def
:=[TT >: This, B](b: B)(implicit op: operators.OpSet.InPlaceImpl2[TT, B]): This
Mutates this by element-wise assignment of b into this.
Mutates this by element-wise assignment of b into this.
- Definition Classes
- NumericOps
-
final
def
:==[TT >: This, B, That](b: B)(implicit op: operators.OpEq.Impl2[TT, B, That]): That
Element-wise equality comparator of this and b.
Element-wise equality comparator of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
:^=[TT >: This, B](b: B)(implicit op: operators.OpPow.InPlaceImpl2[TT, B]): This
Mutates this by element-wise exponentiation of this by b.
Mutates this by element-wise exponentiation of this by b.
- Definition Classes
- NumericOps
-
final
def
:^^=[TT >: This, B](b: B)(implicit op: operators.OpXor.InPlaceImpl2[TT, B]): This
Mutates this by element-wise xor of this and b.
Mutates this by element-wise xor of this and b.
- Definition Classes
- NumericOps
-
final
def
:|=[TT >: This, B](b: B)(implicit op: operators.OpOr.InPlaceImpl2[TT, B]): This
Mutates this by element-wise or of this and b.
Mutates this by element-wise or of this and b.
- Definition Classes
- NumericOps
-
final
def
<:<[TT >: This, B, That](b: B)(implicit op: operators.OpLT.Impl2[TT, B, That]): That
Element-wise less=than comparator of this and b.
Element-wise less=than comparator of this and b.
- Definition Classes
- NumericOps
-
final
def
<:=[TT >: This, B, That](b: B)(implicit op: operators.OpLTE.Impl2[TT, B, That]): That
Element-wise less-than-or-equal-to comparator of this and b.
Element-wise less-than-or-equal-to comparator of this and b.
- Definition Classes
- NumericOps
-
final
def
==(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
-
final
def
>:=[TT >: This, B, That](b: B)(implicit op: operators.OpGTE.Impl2[TT, B, That]): That
Element-wise greater-than-or-equal-to comparator of this and b.
Element-wise greater-than-or-equal-to comparator of this and b.
- Definition Classes
- NumericOps
-
final
def
>:>[TT >: This, B, That](b: B)(implicit op: operators.OpGT.Impl2[TT, B, That]): That
Element-wise greater-than comparator of this and b.
Element-wise greater-than comparator of this and b.
- Definition Classes
- NumericOps
-
def
\[TT >: This, B, That](b: B)(implicit op: operators.OpSolveMatrixBy.Impl2[TT, B, That]): That
Shaped solve of this by b.
Shaped solve of this by b.
- Definition Classes
- ImmutableNumericOps
-
final
def
^:^[TT >: This, B, That](b: B)(implicit op: operators.OpPow.Impl2[TT, B, That]): That
Element-wise exponentiation of this and b.
Element-wise exponentiation of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
^^[TT >: This, B, That](b: B)(implicit op: operators.OpXor.Impl2[TT, B, That]): That
Alias for :^^(b) for all b.
Alias for :^^(b) for all b.
- Definition Classes
- ImmutableNumericOps
-
final
def
^^:^^[TT >: This, B, That](b: B)(implicit op: operators.OpXor.Impl2[TT, B, That]): That
Element-wise logical "xor" operator -- returns true if only one of the corresponding elements is non-zero.
Element-wise logical "xor" operator -- returns true if only one of the corresponding elements is non-zero.
- Definition Classes
- ImmutableNumericOps
-
final
def
^^=[TT >: This, B](b: B)(implicit op: operators.OpXor.InPlaceImpl2[TT, B]): This
Mutates this by element-wise xor of this and b.
Mutates this by element-wise xor of this and b.
- Definition Classes
- NumericOps
- def active: TensorActive[K, V, This]
-
def
apply[Slice1, Slice2, Result](slice1: Slice1, slice2: Slice2)(implicit canSlice: CanSlice2[This, Slice1, Slice2, Result]): Result
Method for slicing that is tuned for Matrices.
-
def
apply[Result](a: K, slice: K*)(implicit canSlice: CanSlice[This, Seq[K], Result]): Result
Slice a sequence of elements.
Slice a sequence of elements. Must be at least 2.
-
def
apply[Slice, Result](slice: Slice)(implicit canSlice: CanSlice[This, Slice, Result]): Result
method for slicing a tensor.
method for slicing a tensor. For instance, DenseVectors support efficient slicing by a Range object.
-
final
def
asInstanceOf[T0]: T0
- Definition Classes
- Any
-
def
clone(): AnyRef
- Attributes
- protected[java.lang]
- Definition Classes
- AnyRef
- Annotations
- @throws( ... )
-
final
def
dot[TT >: This, B, BB >: B, That](b: B)(implicit op: operators.OpMulInner.Impl2[TT, BB, That]): That
Inner product of this and b.
Inner product of this and b.
- Definition Classes
- ImmutableNumericOps
-
final
def
eq(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
-
def
equals(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
-
def
finalize(): Unit
- Attributes
- protected[java.lang]
- Definition Classes
- AnyRef
- Annotations
- @throws( classOf[java.lang.Throwable] )
-
def
findAll(f: (V) ⇒ Boolean): IndexedSeq[K]
Returns all indices k whose value satisfies a predicate.
Returns all indices k whose value satisfies a predicate.
- Definition Classes
- QuasiTensor
-
def
forall(fn: (V) ⇒ Boolean): Boolean
Returns true if and only if the given predicate is true for all elements.
-
def
forall(fn: (K, V) ⇒ Boolean): Boolean
Returns true if and only if the given predicate is true for all elements.
-
def
foreachKey[U](fn: (K) ⇒ U): Unit
Applies the given function to each key in the tensor.
-
def
foreachPair[U](fn: (K, V) ⇒ U): Unit
Applies the given function to each key and its corresponding value.
-
def
foreachValue[U](fn: (V) ⇒ U): Unit
Applies the given function to each value in the map (one for each element of the domain, including zeros).
-
final
def
getClass(): Class[_]
- Definition Classes
- AnyRef → Any
-
def
hashCode(): Int
- Definition Classes
- QuasiTensor → AnyRef → Any
-
final
def
isInstanceOf[T0]: Boolean
- Definition Classes
- Any
- def keys: TensorKeys[K, V, This]
-
def
mapActivePairs[TT >: This, O, That](f: (K, V) ⇒ O)(implicit bf: CanMapKeyValuePairs[TT, K, V, O, That]): That
Maps all active key-value pairs values.
-
def
mapActiveValues[TT >: This, O, That](f: (V) ⇒ O)(implicit bf: CanMapActiveValues[TT, V, O, That]): That
Maps all non-zero values.
-
def
mapPairs[TT >: This, O, That](f: (K, V) ⇒ O)(implicit bf: CanMapKeyValuePairs[TT, K, V, O, That]): That
Creates a new map containing a transformed copy of this map.
-
def
mapValues[TT >: This, O, That](f: (V) ⇒ O)(implicit bf: CanMapValues[TT, V, O, That]): That
Creates a new map containing a transformed copy of this map.
-
final
def
ne(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
-
final
def
notify(): Unit
- Definition Classes
- AnyRef
-
final
def
notifyAll(): Unit
- Definition Classes
- AnyRef
- def pairs: TensorPairs[K, V, This]
-
final
def
synchronized[T0](arg0: ⇒ T0): T0
- Definition Classes
- AnyRef
-
final
def
t[TT >: This, That, Slice1, Result](a: Slice1)(implicit op: CanTranspose[TT, That], canSlice: CanSlice[That, Slice1, Result]): Result
A transposed view of this object, followed by a slice.
A transposed view of this object, followed by a slice. Sadly frequently necessary.
- Definition Classes
- ImmutableNumericOps
-
final
def
t[TT >: This, That, Slice1, Slice2, Result](a: Slice1, b: Slice2)(implicit op: CanTranspose[TT, That], canSlice: CanSlice2[That, Slice1, Slice2, Result]): Result
A transposed view of this object, followed by a slice.
A transposed view of this object, followed by a slice. Sadly frequently necessary.
- Definition Classes
- ImmutableNumericOps
-
final
def
t[TT >: This, That](implicit op: CanTranspose[TT, That]): That
A transposed view of this object.
A transposed view of this object.
- Definition Classes
- ImmutableNumericOps
-
def
toString(): String
- Definition Classes
- AnyRef → Any
-
final
def
unary_: That
- Definition Classes
- ImmutableNumericOps
-
final
def
unary_-[TT >: This, That](implicit op: operators.OpNeg.Impl[TT, That]): That
- Definition Classes
- ImmutableNumericOps
- def values: TensorValues[K, V, This]
-
final
def
wait(): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws( ... )
-
final
def
wait(arg0: Long, arg1: Int): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws( ... )
-
final
def
wait(arg0: Long): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws( ... )
-
final
def
|[TT >: This, B, That](b: B)(implicit op: operators.OpOr.Impl2[TT, B, That]): That
Alias for :||(b) for all b.
Alias for :||(b) for all b.
- Definition Classes
- ImmutableNumericOps
-
final
def
|:|[TT >: This, B, That](b: B)(implicit op: operators.OpOr.Impl2[TT, B, That]): That
Element-wise logical "or" operator -- returns true if either element is non-zero.
Element-wise logical "or" operator -- returns true if either element is non-zero.
- Definition Classes
- ImmutableNumericOps
-
final
def
|=[TT >: This, B](b: B)(implicit op: operators.OpOr.InPlaceImpl2[TT, B]): This
Mutates this by element-wise or of this and b.
Mutates this by element-wise or of this and b.
- Definition Classes
- NumericOps
Deprecated Value Members
-
final
def
:%[TT >: This, B, That](b: B)(implicit op: operators.OpMod.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use %:% instead.
-
final
def
:&[TT >: This, B, That](b: B)(implicit op: operators.OpAnd.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use &:& instead.
-
final
def
:*[TT >: This, B, That](b: B)(implicit op: operators.OpMulScalar.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use *:* instead.
-
final
def
:+[TT >: This, B, That](b: B)(implicit op: operators.OpAdd.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use +:+ instead.
-
final
def
:-[TT >: This, B, That](b: B)(implicit op: operators.OpSub.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use -:- instead.
-
final
def
:/[TT >: This, B, That](b: B)(implicit op: operators.OpDiv.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use /:/ instead.
-
final
def
:<[TT >: This, B, That](b: B)(implicit op: operators.OpLT.Impl2[TT, B, That]): That
- Definition Classes
- NumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use <:< instead.
-
final
def
:<=[TT >: This, B, That](b: B)(implicit op: operators.OpLTE.Impl2[TT, B, That]): That
- Definition Classes
- NumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use <:= instead.
-
final
def
:>[TT >: This, B, That](b: B)(implicit op: operators.OpGT.Impl2[TT, B, That]): That
- Definition Classes
- NumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use >:> instead.
-
final
def
:>=[TT >: This, B, That](b: B)(implicit op: operators.OpGTE.Impl2[TT, B, That]): That
- Definition Classes
- NumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use >:= instead.
-
final
def
:^[TT >: This, B, That](b: B)(implicit op: operators.OpPow.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use : instead.
-
final
def
:^^[TT >: This, B, That](b: B)(implicit op: operators.OpXor.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use : instead.
-
final
def
:|[TT >: This, B, That](b: B)(implicit op: operators.OpOr.Impl2[TT, B, That]): That
- Definition Classes
- ImmutableNumericOps
- Annotations
- @deprecated
- Deprecated
(Since version 0.13) This operator has confusing and often surprising precedence that leads to bugs. Use |:| instead.
-
def
all(implicit semi: Semiring[V]): Boolean
Returns true if all elements are non-zero
Returns true if all elements are non-zero
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use breeze.linalg.all instead
-
def
any(implicit semi: Semiring[V]): Boolean
Returns true if some element is non-zero
Returns true if some element is non-zero
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use breeze.linalg.any instead
-
def
argmax(implicit ord: Ordering[V]): K
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use argmax(t) instead of t.argmax
-
def
argmin(implicit ord: Ordering[V]): K
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use argmin(t) instead of t.argmin
-
def
argsort(implicit ord: Ordering[V]): IndexedSeq[K]
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use argsort(t) instead of t.argsort
-
def
argtopk(k: Int)(implicit ordering: Ordering[V]): IndexedSeq[K]
Returns the k indices with maximum value.
Returns the k indices with maximum value. (NOT absolute value.)
- k
how many to return
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use argtopk(t, k) instead of t.argtopk(k)
-
def
forallValues(fn: (V) ⇒ Boolean): Boolean
Returns true if and only if the given predicate is true for all elements.
Returns true if and only if the given predicate is true for all elements.
- Annotations
- @deprecated
- Deprecated
(Since version 0.8) Please use 'forall' with the same arguments, which is more in accordance with scala.collections syntax
-
def
max(implicit ord: Ordering[V]): V
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use max(t) instead of t.max
-
def
min(implicit ord: Ordering[V]): V
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use min(t) instead of t.min
-
def
sum(implicit num: Numeric[V]): V
- Definition Classes
- QuasiTensor
- Annotations
- @deprecated
- Deprecated
(Since version 0.6) Use sum(t) instead of t.sum