FoldLeftBy

final class FoldLeftBy[A, B, R](by: A => B)(initial: R, f: (R, B) => R) extends Aggregation[A]
trait Aggregation[A]
trait Serializable
class Object
trait Matchable
class Any

Type members

Types

override type Out = R

Value members

Concrete methods

override def apply(xs: Iterable[A]): R
Definition Classes

Inherited methods

def &&[A0 <: A](that: Aggregation[A0])(implicit tupled: TupleFlatten[(Out, Out)]): Of[A0, Out]
Inherited from:
Aggregation
def contramap[A0](f: A0 => A): Of[A0, Out]
Inherited from:
Aggregation
def map[B](f: Out => B): Of[A, B]
Inherited from:
Aggregation
final override def processWindow(order: Ordering[A], values: Iterable[A])(implicit flatten: TupleFlatten[(A, Out)]): Iterable[Out]
Definition Classes
Inherited from:
Aggregation