Contramapped

final class Contramapped[A0, A, B](base: Of[A, B], f: A0 => A) extends Aggregation[A0]
trait Aggregation[A0]
trait QueryExpression[A0]
trait Serializable
class Object
trait Matchable
class Any

Type members

Types

override type Out = B

Value members

Concrete methods

override def apply(xs: Iterable[A0]): B
Definition Classes

Inherited methods

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