|
Scala Library Documentation
|
|
scala/Function1.scala]
trait
Function1[-T1, +R]
extends AnyRefFunction with 1 parameters.
In the following example the definition of
succ is a shorthand for the anonymous class definition
anonfun1:
object Main extends Application {
val succ = (x: Int) => x + 1
val anonfun1 = new Function1[Int, Int] {
def apply(x: Int): Int = x + 1
}
Console.println(succ(0))
Console.println(anonfun1(0))
}| Method Summary | |
def
|
andThen
[A](g : (R) => A) : (T1) => A
(f andThen g)(x) = g(f(x))
|
abstract def
|
apply (v1 : T1) : R |
def
|
compose
[A](g : (A) => T1) : (A) => R
(f compose g)(x) = f(g(x))
|
override def
|
toString : String |
| Methods inherited from AnyRef | |
| getClass, hashCode, equals, clone, notify, notifyAll, wait, wait, wait, finalize, ==, !=, eq, ne, synchronized |
| Methods inherited from Any | |
| ==, !=, isInstanceOf, asInstanceOf |
| Method Details |
|
Scala Library Documentation
|
|