Aggregation

trait Aggregation[-A] extends QueryExpression[A]
Companion:
object
trait Serializable
class Object
trait Matchable
class Any
class Avg[A]
class AvgBy[A, B]
class Chained[A, Out0, Out1, U]
class Const[A]
class Contramapped[A0, A, B]
class Count[A]
class Distinct[A]
class DistinctBy[A, B]
class FlatDistinctBy[A, B]
class FoldLeft[A, B]
class FoldLeftBy[A, B, R]
class Mapped[A, Out0, B]
class Max[A]
class MaxOf[A, B]
class Min[A]
class MinOf[A, B]
class Product[A]
class ProductBy[A, B]
class Reduce[A]
class ReduceBy[A, B]
class Report1[A, B, U1]
class Report2[A, B, C, U1, U2]
class Std[A]
class StdBy[A, B]
class Sum[A]
class SumBy[A, B]
class ToList[A]
class ToListBy[A, B]

Type members

Inherited types

type Out
Inherited from:
QueryExpression

Value members

Abstract methods

def apply(values: Iterable[A]): Out

Concrete methods

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