Const

final class Const[A](value: A) extends Aggregation[Any]
trait Aggregation[Any]
trait QueryExpression[Any]
trait Serializable
class Object
trait Matchable
class Any

Type members

Types

override type Out = A

Value members

Concrete methods

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

Inherited methods

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