Lebesgue measure: Difference between revisions

From formulasearchengine
Jump to navigation Jump to search
en>Tobias Bergemann
Reverted 1 edit by 61.3.169.251 (talk). (TW)
en>FrescoBot
m Bot: link syntax and minor changes
 
Line 1: Line 1:
[[File:Greek lc lamda thin.svg|thumb|right|150px|The lowercase [[lambda]], the 11th letter of the [[Greek alphabet]], is used to symbolize the lambda calculus.]]
Greetings. The author's name is Kourtney but she doesn't like when people use her full [http://Www.Twitpic.com/tag/identity identity]. Her husband doesn't so [http://answers.Yahoo.com/search/search_result?p=comprehensive&submit-go=Search+Y!+Answers comprehensive] the way she does but what she really likes doing is jogging and she'll be starting something else along with it. He works as a payroll sales person. Vermont is lifting place I've been residing in and Vehicles every day living at this site. Go to my web site find out more: http://dcfm.ca/xe/index.php?mid=news&listStyle=webzine&document_srl=1041097<br><br>My web-site :: [http://dcfm.ca/xe/index.php?mid=news&listStyle=webzine&document_srl=1041097 nicki minaj and lil wayne sex tape online]
'''Lambda calculus''' (also written as '''λ-calculus''') is a [[formal system]] in [[mathematical logic]] and [[computer science]] for expressing [[computability|computation]] based on function [[Abstraction (computer science)|abstraction]] and [[function application|application]] using variable [[Name binding|binding]] and [[Substitution (algebra)|substitution]]. First formulated by [[Alonzo Church]] to formalize the concept of [[Computable function|effective computability]], lambda calculus found early successes in the area of [[computability theory]], such as a negative answer to [[David Hilbert|Hilbert]]'s [[Entscheidungsproblem]]. Lambda calculus is a conceptually simple [[Turing completeness|universal model of computation]] (Turing showed in 1937<ref>A. M. Turing, "Computability and λ-Definability", The Journal of Symbolic Logic, Vol. 2, No. 4. (Dec., 1937), pp. 153-163.</ref> that [[Turing machine]]s equalled the lambda calculus in expressiveness). The name derives from the Greek letter lambda (λ) used to denote [[Free variables and bound variables|binding]] a variable in a function.
 
Because of the importance of the notion of variable binding and substitution, there is not just one system of lambda calculus, and in particular there are ''typed'' and ''untyped'' variants. Historically, the most important system was the untyped lambda calculus, in which function application has no restrictions (so the notion of the [[domain of a function]] is not built into the system). In the [[Church–Turing thesis|Church&ndash;Turing Thesis]], the untyped lambda calculus is claimed to be capable of computing all [[effective method|effectively calculable]] functions. The typed lambda calculus is a variety that restricts function application, so that functions can only be applied if they are capable of accepting the given input's "type" of data.
 
Today, the lambda calculus has applications in many different areas in [[mathematics]], [[philosophy]],<ref>Coquand, Thierry, "Type Theory", The Stanford Encyclopedia of Philosophy  (Summer 2013 Edition), Edward N. Zalta (ed.), URL = <http://plato.stanford.edu/archives/sum2013/entries/type-theory/>.</ref> [[linguistics]],<ref>{{Citation|url=http://books.google.co.uk/books?id=9CdFE9X_FCoC |title=Categorial Investigations: Logical and Linguistic Aspects of the Lambek Calculus - Michael Moortgat - Google Books |publisher=Books.google.co.uk |date= 1988-01-01|accessdate=2013-09-15|isbn=9789067653879}}</ref><ref>{{Citation|url=http://books.google.co.uk/books?id=nyFa5ngYThMC |title=Computing Meaning - Google Books |publisher=Books.google.co.uk |date= 2008-07-02|accessdate=2013-09-15|isbn=9781402059575}}</ref> and [[computer science]]. It is still used in the area of computability theory, although [[Turing machines]] are also an important model for computation. Lambda calculus has played an important role in the development of the [[Programming language theory|theory of programming languages]]. Counterparts to lambda calculus in computer science are [[functional programming language]]s, which essentially implement the calculus (augmented with some [[Constant (programming)|constants]] and [[datatype]]s). Beyond programming languages, the lambda calculus also has many applications in [[proof theory]]. A major example of this is the [[Curry&ndash;Howard correspondence]], which gives a correspondence between different systems of typed lambda calculus and systems of [[formal logic]].
 
==Lambda calculus in history of mathematics==
The lambda calculus was introduced by mathematician [[Alonzo Church]] in the 1930s as part of an investigation into the [[foundations of mathematics]].<ref>A. Church, "A set of postulates for the foundation of logic", ''Annals of Mathematics'', Series 2, 33:346–366 (1932).</ref><ref>For a full history, see Cardone and Hindley's "History of Lambda-calculus and Combinatory Logic" (2006).</ref>  The original system was shown to be [[Consistency|logically inconsistent]] in 1935 when [[Stephen Kleene]] and [[J. B. Rosser]] developed the [[Kleene&ndash;Rosser paradox]].
 
Subsequently, in 1936 Church isolated and published just the portion relevant to computation, what is now called the untyped lambda calculus.<ref>A. Church, "An unsolvable problem of elementary number theory", ''American Journal of Mathematics'', Volume 58, No. 2. (April 1936), pp. 345-363.</ref> In 1940, he also introduced a computationally weaker, but logically consistent system, known as the [[simply typed lambda calculus]].<ref>A. Church, "A Formulation of the Simple Theory of Types", ''Journal of Symbolic Logic'', Volume 5 (1940).</ref>
 
==Informal description==
{{no footnotes|section|date=September 2013}}
 
===Motivation===
[[Computable function]]s are a fundamental concept within computer science and mathematics. The λ-calculus provides a simple [[Semantics#Computer science|semantics]] for computation, enabling properties of computation to be studied formally. The λ-calculus incorporates two simplifications that make this semantics simple.
 
One first simplification is that the λ-calculus treats functions "anonymously", without giving them explicit names. For example, the function
:<math>\operatorname{sqsum}(x, y) = x \times x + y \times y</math>
can be rewritten in ''[[Anonymous function|anonymous form]]'' as
:<math>(x, y) \mapsto x \times x + y \times y</math>
(read as "the pair of <math>x</math> and <math>y</math> is mapped to <math>x \times x + y \times y</math>"). Similarly,
:<math>\operatorname{id}(x) = x</math>
can be rewritten in anonymous form as <math>x \mapsto x</math>, where the input is simply mapped to itself.
 
The second simplification is that the λ-calculus only uses functions of a single input. An ordinary function that requires two inputs, for instance the <math>\operatorname{sqsum}</math> function, can be reworked into an equivalent function that accepts a single input, and as output returns ''another'' function, that in turn accepts a single input. For example,
:<math>(x, y) \mapsto x \times x + y \times y</math>
can be reworked into
:<math>x \mapsto (y \mapsto x \times x + y \times y)</math>
This method, known as [[currying]], transforms a function that takes multiple arguments into a chain of functions each with a single argument.
 
[[Function application]] of the <math>\operatorname{sqsum}</math> function to the arguments (5, 2), yields at once
:<math>((x, y) \mapsto x \times x + y \times y)(5, 2)</math>
:<math> = 5 \times 5 + 2 \times 2 </math>
:<math> = 29</math>,
whereas evaluation of the curried version requires one more step
:<math>((x \mapsto (y \mapsto x \times x + y \times y))(5))(2)</math>
:<math> = (y \mapsto 5 \times 5 + y \times y)(2)</math>
:<math> = 5 \times 5 + 2 \times 2</math>
:<math> = 29</math>
to arrive at the same result.
 
===The lambda calculus===
The lambda calculus consists of a language of '''lambda terms''', which is defined by a certain formal syntax, and a set of transformation rules, which allow manipulation of the lambda terms. These transformation rules can be viewed as an equational theory or as an [[operational definition]].
 
As described above, all functions in the lambda calculus are [[anonymous function]]s, having no names. They only accept one input variable, with currying used to implement functions with several variables.
 
====Lambda terms====
 
The syntax of the lambda calculus defines some expressions as valid lambda calculus expression and some as invalid, just as some strings of characters are valid [[C (programming language)|C]] programs and some are not. A valid lambda calculus expression is called a "lambda term".
 
The following three rules give an [[inductive definition]] that can be applied to build all syntactically valid lambda terms:
* a variable, <math>x</math>, is itself a valid lambda term
* if <math>t</math> is a lambda term, and <math>x</math> is a variable, then <math>(\lambda x.t)</math> is a lambda term (called a '''lambda abstraction''');
* if <math>t</math> and <math>s</math> are lambda terms, then <math>(ts)</math> is a lambda term (called an '''application''').
Nothing else is a lambda term. Thus a lambda term is valid if and only if it can be obtained by repeated application of these three rules. However, some parentheses can be omitted according to certain rules. For example, the outermost parentheses are usually not written.
 
A '''lambda abstraction''' <math>\lambda x.t</math> is a definition of an anonymous function that is capable of taking a single input <math>x</math> and substituting it into the expression <math>t</math>.
It thus defines an anonymous function that takes x and returns t. For example <math>\lambda x.x^2+2</math> is a lambda abstraction for the function <math>f(x) = x^2 + 2</math> using the term <math>x^2+2</math> for ''t''. The definition of a function with a lambda abstraction merely "sets up" the function but does not invoke it.  The abstraction [[Free variables and bound variables|binds]] the variable <math>x</math> in the term <math>t</math>.
 
An '''application''' <math>ts</math> represents the application of a function <math>t</math> to an input <math>s</math>, that is, it represents the act of calling function ''t'' on input ''s'' to produce <math>t(s)</math>.
 
There is no concept in lambda calculus of variable declaration. In a definition such as <math>\lambda x.x+y</math> (i.e. <math>f(x) = x + y</math>), the lambda calculus treats ''y'' as a variable that is not yet defined. The lambda abstraction <math>\lambda x.x+y</math> is syntactically valid, and represents a function that adds its input to the yet-unknown ''y''.
 
Bracketing may be used and may be needed to disambiguate terms. For example, <math>\lambda x.((\lambda x.x)x)</math> and <math>(\lambda x.(\lambda x.x)) x</math> denote different terms.
 
==== Functions that operate on functions ====
 
In lambda calculus, functions are taken to be '[[First-class object|first class values]]', so functions may be used as the inputs, or be returned as outputs from other functions.
 
For example, <math>\lambda x.x</math> represents the identity function, <math>x \rightarrow x</math>, and <math>(\lambda x.x)y</math> represents the identity function applied to <math>y</math>. Further, <math>(\lambda x.y)</math> represents the '''constant function''' <math>x \rightarrow y</math>, the function that always returns <math>y</math>, no matter the input. In lambda calculus, function application is regarded as [[Operator associativity|left-associative]], so that <math>stx</math> means <math>(st)x</math>.
 
There are several notions of "equivalence" and "reduction" that allow lambda terms to be "reduced" to "equivalent" lambda terms.
 
====Alpha equivalence====
A basic form of equivalence, definable on lambda terms, is alpha equivalence. It captures the intuition that the particular choice of a bound variable, in a lambda abstraction, does not (usually) matter.
For instance, <math>\lambda x.x</math> and <math>\lambda y.y</math> are alpha-equivalent lambda terms, and they both represent the same function (the identity function).
The terms <math>x</math> and <math>y</math> are not alpha-equivalent, because they are not bound in a lambda abstraction.
In many presentations, it is usual to identify alpha-equivalent lambda terms.
 
The following definitions are necessary in order to be able to define beta reduction.
 
====Free variables====
The '''free variables''' of a term are those variables not bound by a lambda abstraction. The set of free variables of an expression is defined inductively:
* The free variables of <math>x</math> are just <math>x</math>
* The set of free variables of <math>\lambda x.t</math> is the set of free variables of <math>t</math>, but with <math>x</math> removed
* The set of free variables of <math>ts</math> are the union of the set of free variables of <math>t</math> and the set of free variables of <math>s</math>.
 
For example, the lambda term representing the identity <math>\lambda x.x</math> has no free variables, but the function <math>\lambda x.x+y</math> has a single free variable, <math>y</math>.
 
====Capture-avoiding substitutions====
 
Suppose <math>t</math>, <math>s</math> and <math>r</math> are lambda terms and <math>x</math> and <math>y</math> are variables.
The notation <math>t[x := r]</math> indicates substitution of <math>r</math> for <math>x</math> in <math>t</math> in a ''capture-avoiding'' manner. This is defined so that:
* <math>x[x := r] = r</math>;
* <math>y[x := r] = y</math> if <math>x \neq y</math>;
* <math>(ts)[x := r] = (t[x := r])(s[x := r])</math>;
* <math>(\lambda x.t)[x := r] = \lambda x.t</math>;
* <math>(\lambda y.t)[x := r] = \lambda y.(t[x := r])</math> if <math>x \neq y</math> and <math>y</math> is not in the free variables of <math>r</math>. The variable <math>y</math> is said to be "fresh" for <math>r</math>.
 
For example, <math>(\lambda x.x)[y := y] = \lambda x.(x[y := y]) = \lambda x.x</math>, and <math>((\lambda x.y)x)[x := y] = ((\lambda x.y)[x := y])(x[x := y]) = (\lambda x.y)y</math>.
 
The freshness condition (requiring that <math>y</math> is not in the free variables of <math>r</math>)  is crucial in order to ensure that substitution does not change the meaning of functions.
For example, a substitution is made that ignores  the freshness condition: <math>(\lambda x.y)[y := x] = \lambda x.(y[y := x]) = \lambda x.x</math>. This substitution turns the constant function <math>\lambda x.y</math> into the identity <math>\lambda x.x</math> by substitution.
 
In general, failure to meet the freshness condition can be remedied by alpha-renaming with a suitable fresh variable.
For example, switching back to our correct notion of substitution, in <math>(\lambda y.x)[x := y]</math> the lambda abstraction can be renamed with a fresh variable <math>z</math>, to obtain <math>(\lambda z.x)[x := y] = \lambda z.(x[x := y]) = \lambda z.y</math>, and the meaning of the function is preserved by substitution.
 
====Beta reduction====
The beta reduction rule states that an application of the form <math>( \lambda x . t) s</math> reduces to the term <math> t [ x := s]</math>. The notation <math>( \lambda x . t ) s \to t [ x := s ] </math> is used to indicate that <math>( \lambda x .t ) s </math> beta reduces to <math> t [ x := s ] </math>.
For example, for every <math>s</math>, <math>( \lambda x . x ) s \to x[ x := s ] = s </math>. This demonstrates that <math> \lambda x . x </math> really is the identity.
Similarly, <math>( \lambda x . y ) s \to y [ x := s ] = y </math>, which demonstrates that <math> \lambda x . y </math> is a constant function.
 
The lambda calculus may be seen as an idealised functional programming language, like [[Haskell (programming language)|Haskell]] or [[Standard ML]].
Under this view, beta reduction corresponds to a computational step. This step can be repeated by additional beta conversions until there are no more applications left to reduce. In the untyped lambda calculus, as presented here, this reduction process may not terminate.
For instance, consider the term <math>( \lambda x . xx)( \lambda x . xx )</math>.
Here <math>( \lambda x . xx)( \lambda x . xx) \to ( xx )[ x := \lambda x . xx ] = ( x [ x := \lambda x . xx ] )( x [ x := \lambda x . xx ] ) = ( \lambda x . xx)( \lambda x . xx )</math>.
That is, the term reduces to itself in a single beta reduction, and therefore the reduction process will never terminate.
 
Another aspect of the untyped lambda calculus is that it does not distinguish between different kinds of data.
For instance, it may be desirable to write a function that only operates on numbers. However, in the untyped lambda calculus, there is no way to prevent a function from being applied to [[truth value]]s,  strings, or other non-number objects.
 
==Formal definition==
 
===Definition===
Lambda expressions are composed of
* variables v<sub>1</sub>, v<sub>2</sub>, ..., v<sub>n</sub>, ...
* the abstraction symbols lambda 'λ' and dot '.'
* parentheses ( )
The set of lambda expressions, Λ, can be [[Recursive definition|defined inductively]]:
#If x is a variable, then x ∈ Λ
#If x is a variable and M ∈ Λ, then (λx.M) ∈ Λ
#If M, N ∈ Λ, then (M N) ∈ Λ
Instances of rule 2 are known as abstractions and instances of rule 3 are known as applications.<ref>{{Citation
  | last = Barendregt
  | first = Hendrik Pieter
  | author-link =
  | last2 =
  | first2 =
  | author2-link =
  | title = The Lambda Calculus: Its Syntax and Semantics
  | place =
  | publisher = North Holland, Amsterdam. [ftp://ftp.cs.ru.nl/pub/CompMath.Found/ErrataLCalculus.pdf Corrections]
  | year = 1984
  | volume = 103
  | series = Studies in Logic and the Foundations of Mathematics
  | edition = Revised
  | url = http://www.elsevier.com/wps/find/bookdescription.cws_home/501727/description
  | doi =
  | id =
  | isbn = 0-444-87508-5}}
</ref>
 
===Notation===
To keep the notation of lambda expressions uncluttered, the following conventions are usually applied.
* Outermost parentheses are dropped: M N instead of (M N)
* Applications are assumed to be left associative: M N P may be written instead of ((M N) P)<ref>{{cite web|url=http://www.lambda-bound.com/book/lambdacalc/node27.html |title=Example for Rules of Associativity |publisher=Lambda-bound.com |date= |accessdate=2012-06-18}}</ref>
* The body of an abstraction extends [[Regular expression#Lazy quantification|as far right as possible]]: λx.M N means λx.(M N) and not (λx.M) N
* A sequence of abstractions is contracted: λx.λy.λz.N is abbreviated as λxyz.N<ref name="Selinger">
{{Citation
  | first = Peter
  | last = Selinger
  | author-link =
  | first2 =
  | last2 =
  | author2-link =
  | editor-last =
  | editor-first =
  | editor2-last =
  | editor2-first =
  | contribution =
  | contribution-url =
  | title = Lecture Notes on the Lambda Calculus
  | year =2008
  | page = 9
  | place =
  | publisher = Department of Mathematics and Statistics, University of Ottawa
  | url = http://www.mathstat.dal.ca/~selinger/papers/lambdanotes.pdf
  | doi =
  | id =
  | bibcode = 2008arXiv0804.3434S
  | volume = 0804
  | arxiv = 0804.3434
  | class = cs.LO }}</ref><ref>{{cite web|url=http://www.lambda-bound.com/book/lambdacalc/node25.html |title=Example for Rule of Associativity |publisher=Lambda-bound.com |date= |accessdate=2012-06-18}}</ref>
 
===Free and bound variables===
The abstraction operator, λ, is said to bind its variable wherever it occurs in the body of the abstraction. Variables that fall within the scope of an abstraction are said to be ''bound''. All other variables are called ''free''. For example, in the following expression y is a bound variable and x is free: <tt>λ''y''.''x'' ''x'' ''y''</tt>. Also note that a variable is bound by its "nearest" abstraction. In the following example the single occurrence of x in the expression is bound by the second lambda: <tt>λ''x''.''y''  (λ''x''.''z'' ''x'')</tt>
 
The set of ''free variables'' of a lambda expression, M, is denoted as FV(M) and is defined by recursion on the structure of the terms, as follows:
# FV(x) = {x}, where x is a variable
# FV(λx.M) = FV(M) \ {x}
# FV(M N) = FV(M) ∪ FV(N)<ref name="BarendregtBarendsen">{{Citation
  | last = Barendregt
  | first = Henk
  | author-link =
  | last2 = Barendsen
  | first2 = Erik
  | author2-link =
  | title = Introduction to Lambda Calculus
  | place =
  | publisher =
  | year = March 2000
  | volume =
  | edition =
  | url = ftp://ftp.cs.ru.nl/pub/CompMath.Found/lambda.pdf
  | doi =
  | id =
  | isbn = }}</ref>
 
An expression that contains no free variables is said to be ''closed''. Closed lambda expressions are also known as combinators and are equivalent to terms in [[combinatory logic]].
 
==Reduction==
The meaning of lambda expressions is defined by how expressions can be reduced.<ref>de Queiroz, Ruy J.G.B. "[http://dx.doi.org/10.1111/j.1746-8361.1988.tb00919.x A Proof-Theoretic Account of Programming and the Role of Reduction Rules.]"  ''Dialectica'' '''42'''(4), pages 265-282, 1988.</ref>
 
There are three kinds of reduction:
* '''α-conversion''': changing bound variables ('''alpha''');
* '''β-reduction''': applying functions to their arguments ('''beta''');
* '''η-conversion''': which captures a notion of extensionality ('''eta''').
We also speak of the resulting equivalences: two expressions are ''β-equivalent'', if they can be β-converted into the same expression, and α/η-equivalence are defined similarly.
 
The term ''redex'', short for ''reducible expression'', refers to subterms that can be reduced by one of the reduction rules. For example, <tt>(λ''x''.M) N</tt> is a beta-redex in expressing N is substituted for x in M; if <tt>''x''</tt> is not free in <tt>M</tt>, <tt>λ''x''.M ''x''</tt> is an eta-redex. The expression to which a redex reduces is called its reduct; using the previous example, the reducts of these expressions are respectively <tt>M[''x'':=N]</tt> and <tt>M</tt>.
 
===α-conversion===
Alpha-conversion, sometimes known as alpha-renaming,<ref>{{Citation |title=Design concepts in programming languages |last1=Turbak |first1=Franklyn |last2=Gifford |first2=David |year=2008 |publisher=MIT press |page=251| isbn=978-0-262-20175-9}}</ref> allows bound variable names to be changed. For example, alpha-conversion of <tt>λ''x''.''x''</tt> might yield <tt>λ''y''.''y''</tt>. Terms that differ only by alpha-conversion are called ''α-equivalent''. Frequently in uses of lambda calculus, α-equivalent terms are considered to be equivalent.
 
The precise rules for alpha-conversion are not completely trivial. First, when alpha-converting an abstraction, the only variable occurrences that are renamed are those that are bound to the same abstraction. For example, an alpha-conversion of <tt>λ''x''.λ''x''.''x''</tt> could result in <tt>λ''y''.λ''x''.''x''</tt>, but it could ''not'' result in <tt>λ''y''.λ''x''.''y''</tt>. The latter has a different meaning from the original.
 
Second, alpha-conversion is not possible if it would result in a variable getting captured by a different abstraction. For example, if we replace <tt>''x''</tt> with <tt>''y''</tt> in <tt>λ''x''.λ''y''.''x''</tt>, we get <tt>λ''y''.λ''y''.''y''</tt>, which is not at all the same.
 
In programming languages with static scope, alpha-conversion can be used to make [[name resolution]] simpler by ensuring that no variable name [[Variable shadowing|masks]] a name in a containing [[scope (programming)|scope]] (see [[Name resolution#Alpha renaming to make name resolution trivial|alpha renaming to make name resolution trivial]]).
 
====Substitution====
Substitution, written <tt>''E''[''V'' := ''R'']</tt>, is the process of replacing all free occurrences of the variable <tt>''V''</tt> in the expression <tt>''E''</tt> with expression <tt>''R''</tt>.
Substitution on terms of the λ-calculus is defined by recursion on the structure of terms, as follows (note: x and y are only variables while M and N are any λ expression).
: <tt>''x''[''x'' := N] &nbsp;&nbsp;&nbsp;&nbsp;&nbsp;&nbsp; &equiv; N</tt>
: <tt>''y''[''x'' := N] &nbsp;&nbsp;&nbsp;&nbsp;&nbsp;&nbsp; &equiv; ''y'', if ''x'' ≠ ''y''</tt>
: <tt>(M<sub>1</sub> M<sub>2</sub>)[''x'' := N]&nbsp;&nbsp;&equiv; (M<sub>1</sub>[''x'' := N]) (M<sub>2</sub>[''x'' := N])</tt>
: <tt>(λ''x''.M)[''x'' := N] &nbsp; &equiv; λ''x''.M</tt>
: <tt>(λ''y''.M)[''x'' := N] &nbsp; &equiv; λ''y''.(M[''x'' := N]), if ''x'' ≠ ''y'', ''provided'' ''y'' ∉ FV(N)</tt>
 
To substitute into a lambda abstraction, it is sometimes necessary to α-convert the expression. For example, it is not correct for <tt>(λ''x''.''y'')[''y'' := ''x'']</tt> to result in <tt>(λ''x''.''x'')</tt>, because the substituted <tt>''x''</tt> was supposed to be free but ended up being bound. The correct substitution in this case is <tt>(λ''z''.''x'')</tt>, up to α-equivalence. Notice that substitution is defined uniquely up to α-equivalence.
 
===&beta;-reduction===
Beta-reduction captures the idea of function application. Beta-reduction is defined in terms of substitution: the beta-reduction of <tt>&nbsp;((λ''V''.''E'') ''E&prime;'')&nbsp;</tt> is <tt>''E''[''V'' := ''E&prime;'']</tt>.
 
For example, assuming some encoding of <tt>2, 7, &times;</tt>, we have the following β-reduction: <tt>((λ''n''.''n''&times;2) 7) </tt>→<tt> 7&times;2</tt>.
 
===&eta;-conversion===
Eta-conversion expresses the idea of [[extensionality]], which in this context is that two functions are the same [[if and only if]] they give the same result for all arguments. Eta-conversion converts between <tt>λ''x''.(''f'' ''x'')</tt> and <tt>''f''</tt> whenever <tt>''x''</tt> does not appear free in <tt>''f''</tt>.
 
== Normal forms and confluence ==
{{Main|Normalization property (abstract rewriting)}}
For the untyped lambda calculus, β-reduction as a [[rewrite system|rewriting rule]] is neither [[strongly normalising]] nor [[weakly normalising]].
 
However, it can be shown that β-reduction is [[confluence (abstract rewriting)|confluent]]. (Of course, we are working up to α-conversion, i.e. we consider two normal forms to be equal, if it is possible to α-convert one into the other.)
 
Therefore, both strongly normalising terms and weakly normalising terms have a unique normal form. For strongly normalising terms, any reduction strategy is guaranteed to yield the normal form, whereas for weakly normalising terms, some reduction strategies may fail to find it.
 
==Encoding datatypes==
{{Main|Church encoding|Mogensen–Scott encoding}}
 
The basic lambda calculus may be used to model booleans, [[arithmetic]], data structures and recursion, as illustrated in the following sub-sections.
 
===Arithmetic in lambda calculus===
There are several possible ways to define the [[natural number]]s in lambda calculus, but by far the most common are the [[Church numeral]]s, which can be defined as follows:
: <tt>0 := λ''f''.λ''x''.''x''</tt>
: <tt>1 := λ''f''.λ''x''.''f'' ''x''</tt>
: <tt>2 := λ''f''.λ''x''.''f'' (''f'' ''x'')</tt>
: <tt>3 := λ''f''.λ''x''.''f'' (''f'' (''f'' ''x''))</tt>
and so on. Or using the alternative syntax presented above in ''[[#Notation|Notation]]'':
 
: <tt>0 := λ''fx''.''x''</tt>
: <tt>1 := λ''fx''.''f'' ''x''</tt>
: <tt>2 := λ''fx''.''f'' (''f'' ''x'')</tt>
: <tt>3 := λ''fx''.''f'' (''f'' (''f'' ''x''))</tt>
 
A Church numeral is a [[higher-order function]]—it takes a single-argument function <tt>''f''</tt>, and returns another single-argument function. The Church numeral <tt>''n''</tt> is a function that takes a function <tt>''f''</tt> as argument and returns the <tt>''n''</tt>-th composition of <tt>''f''</tt>, i.e. the function <tt>''f''</tt> composed with itself <tt>''n''</tt> times. This is denoted <tt>''f''<sup>(''n'')</sup></tt> and is in fact the <tt>''n''</tt>-th power of <tt>''f''</tt> (considered as an operator); <tt>''f''<sup>(0)</sup></tt> is defined to be the identity function. Such repeated compositions (of a single function <tt>''f''</tt>) obey the [[laws of exponents]], which is why these numerals can be used for arithmetic. (In Church's original lambda calculus, the formal parameter of a lambda expression was required to occur at least once in the function body, which made the above definition of <tt>0</tt> impossible.)
 
We can define a successor function, which takes a number <tt>''n''</tt> and returns <tt>''n'' + 1</tt> by adding an additional application of <tt>''f''</tt>,where '(mf)x' means the function 'f' is applied 'm' times on 'x':
: <tt>SUCC := λ''n''.λ''f''.λ''x''.''f'' (''n'' ''f'' ''x'')</tt>
Because the <tt>''m''</tt>-th composition of <tt>''f''</tt> composed with the <tt>''n''</tt>-th composition of <tt>''f''</tt> gives the <tt>''m''+''n''</tt>-th composition of <tt>''f''</tt>, addition can be defined as follows:
: <tt>PLUS := λ''m''.λ''n''.λ''f''.λ''x''.''m'' ''f'' (''n'' ''f'' ''x'')</tt>
<tt>PLUS</tt> can be thought of as a function taking two natural numbers as arguments and returning a natural number; it can be verified that
: <tt>PLUS 2 3</tt>
and
: <tt>5</tt>
are equivalent lambda expressions. Since adding <tt>''m''</tt> to a number <tt>''n''</tt> can be accomplished by adding 1 <tt>''m''</tt> times, an equivalent definition is:
: <tt>PLUS := λ''m''.λ''n''.''m'' SUCC ''n''</tt><ref>{{Citation
  | last1 = Felleisen
  | first1 = Matthias
  | last2 = Flatt
  | first2 = Matthew
  | authorlink =
  | title = Programming Languages and Lambda Calculi
  | publisher =
  | year = 2006
  | location =
  | page = 26
  | url = http://www.cs.utah.edu/plt/publications/pllc.pdf
  | doi =
  | id =
  | isbn = }}</ref>
Similarly, multiplication can be defined as
: <tt>MULT := λ''m''.λ''n''.λ''f''.''m'' (''n'' ''f'')</tt><ref>
{{Citation
  | first = Peter
  | last = Selinger
  | author-link =
  | first2 =
  | last2 =
  | author2-link =
  | editor-last =
  | editor-first =
  | editor2-last =
  | editor2-first =
  | contribution =
  | contribution-url =
  | title = Lecture Notes on the Lambda Calculus
  | year =2008
  | page = 16
  | place =
  | publisher = Department of Mathematics and Statistics, University of Ottawa
  | url = http://www.mathstat.dal.ca/~selinger/papers/lambdanotes.pdf
  | doi =
  | id =
  | bibcode = 2008arXiv0804.3434S
  | volume = 0804
  | arxiv = 0804.3434
  | class = cs.LO }}</ref>
Alternatively
: <tt>MULT := λ''m''.λ''n''.''m'' (PLUS ''n'') 0</tt>
since multiplying <tt>''m''</tt> and <tt>''n''</tt> is the same as repeating the add <tt>''n''</tt> function <tt>''m''</tt> times and then applying it to zero.
Exponentiation has a rather simple rendering in Church numerals, namely
: <tt>POW := λ''b''.λ''e''.''e'' ''b''</tt>
The predecessor function defined by <tt>PRED ''n'' = ''n'' − 1</tt> for a positive integer <tt>''n''</tt> and <tt>PRED 0 = 0</tt> is considerably more difficult. The formula
: <tt>PRED := λ''n''.λ''f''.λ''x''.''n'' (λ''g''.λ''h''.''h'' (''g'' ''f'')) (λ''u''.''x'') (λ''u''.''u'')</tt>
can be validated by showing inductively that if ''T'' denotes <tt>(λ''g''.λ''h''.''h'' (''g'' ''f''))</tt>, then <tt>T<sup>(''n'')</sup>(λ''u''.''x'') = (λ''h''.''h''(''f''<sup>(''n''−1)</sup>(''x'')))</tt> for <tt>''n'' > 0</tt>. Two other definitions of <tt>PRED</tt> are given below, one using [[#Logic and predicates|conditionals]] and the other using [[#Pairs|pairs]]. With the predecessor function, subtraction is straightforward. Defining
: <tt>SUB := λ''m''.λ''n''.''n'' PRED ''m''</tt>,
<tt>SUB ''m'' ''n''</tt> yields <tt>''m'' − ''n''</tt> when <tt>''m'' > ''n''</tt> and <tt>0</tt> otherwise.
 
===Logic and predicates===
By convention, the following two definitions (known as Church booleans) are used for the boolean values <tt>TRUE</tt> and <tt>FALSE</tt>:
: <tt>TRUE := λ''x''.λ''y''.''x''</tt>
: <tt>FALSE := λ''x''.λ''y''.''y''</tt>
::(Note that <tt>FALSE</tt> is equivalent to the Church numeral zero defined above)
Then, with these two λ-terms, we can define some logic operators (these are just possible formulations; other expressions are equally correct):
: <tt>AND := λ''p''.λ''q''.''p'' ''q'' ''p''</tt>
: <tt>OR := λ''p''.λ''q''.''p'' ''p'' ''q''</tt>
: <tt>NOT := λ''p''.λ''a''.λ''b''.''p'' ''b'' ''a''</tt>
: <tt>IFTHENELSE := λ''p''.λ''a''.λ''b''.''p'' ''a'' ''b''</tt>
We are now able to compute some logic functions, for example:
 
: <tt>AND TRUE FALSE</tt>
::<tt>≡ (λ''p''.λ''q''.''p'' ''q'' ''p'') TRUE FALSE →<sub>β</sub> TRUE FALSE TRUE</tt>
::<tt>≡ (λ''x''.λ''y''.''x'') FALSE TRUE →<sub>β</sub>  FALSE</tt>
and we see that <tt>AND TRUE FALSE</tt> is equivalent to <tt>FALSE</tt>.
 
A ''predicate'' is a function that returns a boolean value. The most fundamental predicate is <tt>ISZERO</tt>, which returns <tt>TRUE</tt> if its argument is the Church numeral <tt>0</tt>, and <tt>FALSE</tt> if its argument is any other Church numeral:
: <tt>ISZERO := λ''n''.''n'' (λ''x''.FALSE) TRUE</tt>
The following predicate tests whether the first argument is less-than-or-equal-to the second:
: <tt>LEQ := λ''m''.λ''n''.ISZERO (SUB ''m'' ''n'')</tt>,
and since <tt>''m'' = ''n''</tt>, if <tt>LEQ ''m'' ''n''</tt> and <tt>LEQ ''n'' ''m''</tt>, it is straightforward to build a predicate for numerical equality.
 
The availability of predicates and the above definition of <tt>TRUE</tt> and <tt>FALSE</tt> make it convenient to write "if-then-else" expressions in lambda calculus. For example, the predecessor function can be defined as:
: <tt>PRED := λ''n''.''n'' (λ''g''.λ''k''.ISZERO (''g'' 1) ''k'' (PLUS (''g'' ''k'') 1)) (λ''v''.0) 0 </tt>
which can be verified by showing inductively that <tt>''n'' (λ''g''.λ''k''.ISZERO (''g'' 1) ''k'' (PLUS (''g'' ''k'') 1)) (λ''v''.0)</tt> is the add <tt>''n''</tt> − 1 function for <tt>''n''</tt> > 0.
 
===Pairs===
A pair (2-tuple) can be defined in terms of <tt>TRUE</tt> and <tt>FALSE</tt>, by using the [[Church encoding#Church pairs|Church encoding for pairs]]. For example, <tt>PAIR</tt> encapsulates the pair (<tt>''x''</tt>,<tt>''y''</tt>), <tt>FIRST</tt> returns the first element of the pair, and <tt>SECOND</tt> returns the second.
 
: <tt>PAIR := λ''x''.λ''y''.λ''f''.''f'' ''x'' ''y''</tt>
: <tt>FIRST := λ''p''.''p'' TRUE</tt>
: <tt>SECOND := λ''p''.''p'' FALSE</tt>
: <tt>NIL := λ''x''.TRUE </tt>
: <tt>NULL := λ''p''.''p'' (λ''x''.λ''y''.FALSE)</tt>
 
A linked list can be defined as either NIL for the empty list, or the <tt>PAIR</tt> of an element and a smaller list. The predicate <tt>NULL</tt> tests for the value <tt>NIL</tt>. (Alternatively, with <tt>NIL := FALSE</tt>, the construct <tt>''l'' (λ''h''.λ''t''.λ''z''.deal_with_head_''h''_and_tail_''t'') (deal_with_nil)</tt> obviates the need for an explicit NULL test).
 
As an example of the use of pairs, the shift-and-increment function that maps <tt>(''m'', ''n'')</tt> to <tt>(''n'', ''n'' + 1)</tt> can be defined as
: <tt>Φ := λ''x''.PAIR (SECOND ''x'') (SUCC (SECOND ''x''))</tt>
which allows us to give perhaps the most transparent version of the predecessor function:
: <tt>PRED := λ''n''.FIRST (''n'' Φ (PAIR 0 0)).</tt>
 
===Recursion and fixed points===
{{Main|Fixed-point combinator}}
{{see also|SKI combinator calculus#Self-application_and_recursion}}
[[Recursion]] is the definition of a function using the function itself; on the face of it, lambda calculus does not allow this (we can't refer to a value which is yet to be defined, inside the lambda term defining that same value, as all functions are [[Anonymous function|anonymous]] in lambda calculus). However, this impression is misleading: in&ensp; <tt>(λ''x''.''x'' ''x'') ''y''</tt> &ensp;both ''x''‍&thinsp;‍'s refer to the same lambda term, ''y'', so it is possible for a lambda expression &ndash; here ''y'' &ndash; to be arranged to receive itself as its argument value, through self-application.
 
Consider for instance the [[factorial]] function <tt>F(''n'')</tt> recursively defined by
 
:<tt>F(''n'') = 1, if ''n'' = 0; else ''n'' &times; F(''n'' − 1)</tt>.
 
In the lambda expression which is to represent this function, a ''parameter'' (typically the first one) will be assumed to receive the lambda expression itself as its value, so that calling it &ndash; applying it to an argument &ndash; will amount to recursion. Thus to achieve recursion, the intended-as-self-referencing argument (called <tt>''r''</tt> here) must always be passed to itself within the function body, at a call point:
 
:<tt>G := λ''r''. λ''n''.(1, if ''n'' = 0; else ''n'' &times; (''r'' ''r'' (''n''−1)))</tt>
::: with&ensp; <tt> ''r'' ''r'' ''x'' = F ''x'' = G ''r'' ''x''</tt> &ensp;to hold, so&ensp; <tt>''r'' = G</tt> &ensp;and
:<tt>F := G G = (λ''x''.''x'' ''x'') G</tt>
 
The self-application achieves replication here, passing the function's lambda expression on to the next invocation as an argument value, making it available to be referenced and called there.
 
This solves it but requires re-writing each recursive call as self-application. We would like to have a generic solution, without a need for any re-writes:
 
:<tt>G := λ''r''. λ''n''.(1, if ''n'' = 0; else ''n'' &times; (''r'' (''n''−1)))</tt>
::: with&ensp; <tt> ''r'' ''x'' = F ''x'' = G ''r'' ''x''</tt> &ensp;to hold, so&ensp; <tt>''r'' = G ''r'' =: FIX G</tt> &ensp;and
:<tt>F := FIX G</tt> &ensp;where&ensp; <tt>FIX ''g'' := (''r'' where ''r'' = ''g'' ''r'') = ''g'' (FIX ''g'')</tt>
::: so that&ensp; <tt> FIX G = G (FIX G) = (λ''n''.(1, if ''n'' = 0; else ''n'' &times; ((FIX G) (''n''−1)))) </tt>
 
Given a lambda term with first argument representing recursive call (e.g. <tt>G</tt> here), the [[fixed-point combinator|''fixed-point'' combinator]] <tt>FIX</tt> will return a self-replicating lambda expression representing the recursive function (here, <tt>F</tt>). The function does not need to be explicitly passed to itself at any point, for the self-replication is arranged in advance, when it is created, to be done each time it is called. Thus the original lambda expression <tt>(FIX G)</tt> is re-created inside itself, at call-point, achieving [[self-reference]].
 
In fact, there are many possible definitions for this <tt>FIX</tt> operator, the simplest of them being:
 
:<tt>'''Y''' := λ''g''.(λ''x''.''g'' (''x'' ''x'')) (λ''x''.''g'' (''x'' ''x''))</tt>
 
In the lambda calculus, <tt>'''Y''' ''g''</tt>&thinsp; is a fixed-point of <tt>''g''</tt>, as it expands to:
 
:<tt>'''Y''' ''g''</tt>
:<tt>λ''h''.((λ''x''.''h'' (''x'' ''x'')) (λ''x''.''h'' (''x'' ''x''))) ''g''</tt>
:<tt>(λ''x''.''g'' (''x'' ''x'')) (λ''x''.''g'' (''x'' ''x''))</tt>
:<tt>''g'' ((λ''x''.''g'' (''x'' ''x'')) (λ''x''.''g'' (''x'' ''x'')))</tt>
:<tt>''g'' ('''Y''' ''g'')</tt>
 
Now, to perform our recursive call to the factorial function, we would simply call <tt>('''Y''' G) ''n''</tt>,&nbsp; where ''n'' is the number we are calculating the factorial of. Given ''n'' = 4, for example, this gives:
 
:<tt>('''Y''' G) 4 </tt>
:<tt>G ('''Y''' G) 4 </tt>
:<tt>(λ''r''.λ''n''.(1, if ''n'' = 0; else ''n'' × (''r'' (''n''−1)))) ('''Y''' G) 4</tt>
:<tt>(λ''n''.(1, if ''n'' = 0; else ''n'' × (('''Y''' G) (''n''−1)))) 4</tt>
:<tt>1, if 4 = 0; else 4 × (('''Y''' G) (4−1))</tt>
:<tt>4 × (G ('''Y''' G) (4−1))</tt>
:<tt>4 × ((λ''n''.(1, if ''n'' = 0; else ''n'' × (('''Y''' G) (''n''−1)))) (4−1))</tt>
:<tt>4 × (1, if 3 = 0; else 3 × (('''Y''' G) (3−1)))</tt>
:<tt>4 × (3 × (G ('''Y''' G) (3−1)))</tt>
:<tt>4 × (3 × ((λ''n''.(1, if ''n'' = 0; else ''n'' × (('''Y''' G) (''n''−1)))) (3−1)))</tt>
:<tt>4 × (3 × (1, if 2 = 0; else 2 × (('''Y''' G) (2−1))))</tt>
:<tt>4 × (3 × (2 × (G ('''Y''' G) (2−1))))</tt>
:<tt>4 × (3 × (2 × ((λ''n''.(1, if ''n'' = 0; else ''n'' × (('''Y''' G) (''n''−1)))) (2−1))))</tt>
:<tt>4 × (3 × (2 × (1, if 1 = 0; else 1 × (('''Y''' G) (1−1)))))</tt>
:<tt>4 × (3 × (2 × (1 × (G ('''Y''' G) (1−1)))))</tt>
:<tt>4 × (3 × (2 × (1 × ((λ''n''.(1, if ''n'' = 0; else ''n'' × (('''Y''' G) (''n''−1)))) (1−1)))))</tt>
:<tt>4 × (3 × (2 × (1 × (1, if 0 = 0; else 0 × (('''Y''' G) (0−1))))))</tt>
:<tt>4 × (3 × (2 × (1 × (1))))</tt>
:<tt>24</tt>
 
Every recursively defined function can be seen as a fixed point of some suitably defined function closing over the recursive call with an extra argument, and therefore, using <tt>'''Y'''</tt>, every recursively defined function can be expressed as a lambda expression. In particular, we can now cleanly define the subtraction, multiplication and comparison predicate of natural numbers recursively.
 
===Standard terms===
Certain terms have commonly accepted names:
: {{anchor|I}} <tt>'''I''' := λ''x''.''x''</tt>
: {{anchor|K}} <tt>'''K''' := λ''x''.λ''y''.''x''</tt>
: {{anchor|S}} <tt>'''S''' := λ''x''.λ''y''.λ''z''.''x'' ''z'' (''y'' ''z'') </tt>
: {{anchor|B}} <tt>'''B''' := λ''x''.λ''y''.λ''z''.''x'' (''y'' ''z'') </tt>
: {{anchor|C}} <tt>'''C''' := λ''x''.λ''y''.λ''z''.''x'' ''z'' ''y''</tt>
: {{anchor|W}} <tt>'''W''' := λ''x''.λ''y''.''x'' ''y'' ''y''</tt>
: {{anchor|U}} <tt>'''U''' := λ''x''.''x'' ''x''  </tt>
: {{anchor|omega}} <tt>'''ω''' := λ''x''.''x'' ''x'' </tt>
: {{anchor|Omega}} <tt>'''Ω''' := '''ω ω''' </tt>
: {{anchor|Y}} <tt>'''Y''' := λ''g''.(λ''x''.''g'' (''x'' ''x'')) (λ''x''.''g'' (''x'' ''x''))</tt>
 
== Typed lambda calculi ==
{{main|Typed lambda calculus}}
{{Summarize|from|typed lambda calculus|date=August 2009}}<!-- this was requested by multiple editor on talk -->
A '''typed lambda calculus''' is a typed [[formalism (mathematics)|formalism]] that uses the lambda-symbol (<math>\lambda</math>) to denote anonymous function abstraction. In this context, types are usually objects of a syntactic nature that are assigned to lambda terms; the exact nature of a type depends on the calculus considered (see kinds below). From a certain point of view, typed lambda calculi can be seen as refinements of the [[untyped lambda calculus]] but from another point of view, they can also be considered the more fundamental theory and  ''untyped lambda calculus'' a special case with only one type.
 
Typed lambda calculi are foundational [[programming languages]] and are the base of typed [[functional programming languages]] such as [[ML programming language|ML]] and [[Haskell (programming language)|Haskell]] and, more indirectly, typed [[imperative programming|imperative programming languages]]. Typed lambda calculi play an important role in the design of [[type systems]] for programming languages; here typability usually captures desirable properties of the program, e.g. the program will not cause a memory access violation.
 
Typed lambda calculi are closely related to [[mathematical logic]] and [[proof theory]] via the [[Curry&ndash;Howard isomorphism]] and they can be considered as the [[internal language]] of classes of [[category theory|categories]], e.g. the [[simply typed lambda calculus]] is the language of [[cartesian closed category|Cartesian closed categories]] (CCCs).
 
==Computable functions and lambda calculus==
A function ''F'': '''N''' → '''N''' of [[natural number]]s is a computable function [[if and only if]] there exists a lambda expression ''f'' such that for every pair of ''x'', ''y'' in '''N''', ''F''(''x'')=''y'' if and only if ''f'' <tt>''x''</tt>&nbsp;=<sub>β</sub>&nbsp;<tt>''y''</tt>,&nbsp; where <tt>''x''</tt> and <tt>''y''</tt> are the Church numerals corresponding to ''x'' and ''y'', respectively and =<sub>β</sub> meaning equivalence with beta reduction. This is one of the many ways to define computability; see the [[Church-Turing thesis]] for a discussion of other approaches and their equivalence.
 
==Undecidability of equivalence==
There is no algorithm that takes as input two lambda expressions and outputs <tt>TRUE</tt> or <tt>FALSE</tt> depending on whether or not the two expressions are equivalent. This was historically the first problem for which undecidability could be proven. As is common for a proof of undecidability, the proof shows that no computable function can decide the equivalence. [[Church's thesis]] is then invoked to show that no algorithm can do so.
 
Church's proof first reduces the problem to determining whether a given lambda expression has a ''[[Normalization property (abstract rewriting)|normal]] form''. A normal form is an equivalent expression that cannot be reduced any further under the rules imposed by the form. Then he assumes that this predicate is computable, and can hence be expressed in lambda calculus. Building on earlier work by Kleene and constructing a [[Gödel numbering]] for lambda expressions, he constructs a lambda expression <tt>''e''</tt> that closely follows the proof of [[Gödel's incompleteness theorems|Gödel's first incompleteness theorem]]. If <tt>''e''</tt> is applied to its own Gödel number, a contradiction results.
 
==Lambda calculus and programming languages==
As pointed out by [[Peter Landin]]'s 1965 paper <cite>[http://portal.acm.org/citation.cfm?id=363749&coll=portal&dl=ACM A Correspondence between ALGOL 60 and Church's Lambda-notation]</cite>, sequential [[procedural programming|procedural programming languages]] can be understood in terms of the lambda calculus, which provides the basic mechanisms for procedural abstraction and procedure (subprogram) application.
 
Lambda calculus [[Reification (computer science)|reifies]] "functions" and makes them [[first-class object]]s, which raises implementation complexity when it is implemented.
 
===Anonymous functions===
{{main|Anonymous function}}
For example in [[Lisp (programming language)|Lisp]] the 'square' function can be expressed as a lambda expression as follows:
<!-- Please do not add the same example in different languages to this article, see [[Anonymous function]] for that. Thank you! -->
<source lang="Lisp">
(lambda (x) (* x x))
</source>
 
The above example is an expression that evaluates to a first-class function. The symbol <code>lambda</code> creates an anonymous function, given a list of parameter names, <code>(x)</code> &mdash; just a single argument in this case, and an expression that is evaluated as the body of the function, <code>(* x x)</code>. The Haskell example is identical. [[Anonymous functions]] are sometimes called lambda expressions.
 
For example [[Pascal (programming language)|Pascal]] and many other [[Imperative programming|imperative languages]] have long supported passing [[subprograms]] as [[arguments]] to other subprograms through the mechanism of [[function pointers]]. However, function pointers are not a sufficient condition for functions to be [[First-class function|first class]] datatypes, because a function is a first class datatype if and only if new instances of the function can be created at run-time. And this run-time creation of functions is supported in [[Smalltalk]], and more recently in [[Scala (programming language)|Scala]], [[Eiffel (programming language)|Eiffel]] ("agents") and [[C Sharp (programming language)|C#]] ("delegates"), among others. Compiled languages, such as C++, permit run-time selection (i.e., binding) of a variety of already-compiled functions, which is utilized in lieu of compiling additional machine-code instructions, which is what would be needed by compiled languages to achieve full-fledged run-time creation of new functions.
 
===Reduction strategies===
{{details|Evaluation strategy}}
Whether a term is normalising or not, and how much work needs to be done in normalising it if it is, depends to a large extent on the reduction strategy used. The distinction between reduction strategies relates to the distinction in functional programming languages between [[eager evaluation]] and [[lazy evaluation]].
 
;Full beta reductions: Any redex can be reduced at any time. This means essentially the lack of any particular reduction strategy—with regard to reducibility, "all bets are off".
;Applicative order: The rightmost, innermost redex is always reduced first. Intuitively this means a function's arguments are always reduced before the function itself. Applicative order always attempts to apply functions to normal forms, even when this is not possible.
:Most programming languages (including [[Lisp (programming language)|Lisp]], [[ML (programming language)|ML]] and imperative languages like [[C (programming language)|C]] and [[Java programming language|Java]]) are described as "strict", meaning that functions applied to non-normalising arguments are non-normalising. This is done essentially using applicative order, call by value reduction ([[#Call by value|see below]]), but usually called "eager evaluation".
;Normal order: The leftmost, outermost redex is always reduced first. That is, whenever possible the arguments are substituted into the body of an abstraction before the arguments are reduced.
;Call by name: As normal order, but no reductions are performed inside abstractions. For example <tt>λ''x''.(λ''x''.''x'')''x''</tt> is in normal form according to this strategy, although it contains the redex <tt>(λ''x''.''x'')''x''</tt>.
;Call by value: Only the outermost redexes are reduced: a redex is reduced only when its right hand side has reduced to a value (variable or lambda abstraction).
;Call by need: As normal order, but function applications that would duplicate terms instead name the argument, which is then reduced only "when it is needed". Called in practical contexts "lazy evaluation". In implementations this "name" takes the form of a pointer, with the redex represented by a [[thunk (functional programming)|thunk]].
 
Applicative order is not a normalising strategy. The usual counterexample is as follows: define <tt>'''Ω''' = ωω</tt> where <tt>'''ω''' = λ''x''.''xx''</tt>. This entire expression contains only one redex, namely the whole expression; its reduct is again <tt>'''Ω'''</tt>. Since this is the only available reduction, <tt>'''Ω'''</tt> has no normal form (under any evaluation strategy). Using applicative order, the expression <tt>'''KIΩ''' = (λ''x''.λ''y''.''x'') (λ''x''.''x'')'''Ω'''</tt> is reduced by first reducing <tt>'''Ω'''</tt> to normal form (since it is the rightmost redex), but since <tt>'''Ω'''</tt> has no normal form, applicative order fails to find a normal form for <tt>'''KIΩ'''</tt>.
 
In contrast, normal order is so called because it always finds a normalising reduction, if one exists. In the above example, <tt>'''KIΩ'''</tt> reduces under normal order to ''I'', a normal form. A drawback is that redexes in the arguments may be copied, resulting in duplicated computation (for example, <tt>(λ''x''.''xx'') ((λ''x''.''x'')''y'')</tt> reduces to <tt>((λ''x''.''x'')''y'') ((λ''x''.''x'')''y'')</tt> using this strategy; now there are two redexes, so full evaluation needs two more steps, but if the argument had been reduced first, there would now be none).
 
The positive tradeoff of using applicative order is that it does not cause unnecessary computation, if all arguments are used, because it never substitutes arguments containing redexes and hence never needs to copy them (which would duplicate work). In the above example, in applicative order <tt>(λ''x''.''xx'') ((λ''x''.''x'')''y'')</tt> reduces first to <tt>(λ''x''.''xx'')''y''</tt> and then to the normal order <tt>''yy''</tt>, taking two steps instead of three.
 
Most ''purely'' functional programming languages (notably [[Miranda (programming language)|Miranda]] and its descendents, including [[Haskell (programming language)|Haskell]]), and the proof languages of [[Automated theorem prover|theorem prover]]s, use ''[[lazy evaluation]]'', which is essentially the same as call by need. This is like normal order reduction, but call by need manages to avoid the duplication of work inherent in normal order reduction using ''sharing''. In the example given above, <tt>(λ''x''.''xx'') ((λ''x''.''x'')''y'')</tt> reduces to <tt>((λ''x''.''x'')''y'') ((λ''x''.''x'')''y'')</tt>, which has two redexes, but in call by need they are represented using the same object rather than copied, so when one is reduced the other is too.
 
===A note about complexity===
While the idea of beta reduction seems simple enough, it is not an atomic step, in that it must have a non-trivial cost when estimating [[computational complexity]].<ref>R. Statman, "[http://ieeexplore.ieee.org/xpl/freeabs_all.jsp?arnumber=4567929 The typed &lambda;-calculus is not elementary recursive.]" ''Theoretical Computer Science'', (1979) '''9''' pp73-81.</ref> To be precise, one must somehow find the location of all of the occurrences of the bound variable <tt>''V''</tt> in the expression <tt>''E''</tt>, implying a time cost, or one must keep track of these locations in some way, implying a space cost. A naïve search for the locations of <tt>''V''</tt> in <tt>''E''</tt> is [[Big O notation|''O''(''n'')]] in the length ''n'' of <tt>''E''</tt>. This has led to the study of systems that use [[explicit substitution]]. Sinot's [[director string]]s<ref>F.-R. Sinot. "[http://www.lsv.ens-cachan.fr/~sinot/publis.php?onlykey=sinot-jlc05 Director Strings Revisited: A Generic Approach to the Efficient Representation of Free Variables in Higher-order Rewriting.]" ''Journal of Logic and Computation'' '''15'''(2), pages 201-218, 2005.</ref> offer a way of tracking the locations of free variables in expressions.
 
===Parallelism and concurrency===
The [[Church–Rosser theorem|Church–Rosser]] property of the lambda calculus means that evaluation (β-reduction) can be carried out in ''any order'', even in parallel. This means that various [[evaluation strategy#Nondeterministic strategies|nondeterministic evaluation strategies]] are relevant. However, the lambda calculus does not offer any explicit constructs for [[parallel computing|parallelism]]. One can add constructs such as [[Futures and promises|Futures]] to the lambda calculus. Other [[process calculi]] have been developed for describing communication and concurrency.
 
==Semantics==
The fact that lambda calculus terms act as functions on other lambda calculus terms, and even on themselves, led to questions about the semantics of the lambda calculus. Could a sensible meaning be assigned to lambda calculus terms? The natural semantics was to find a set ''D'' isomorphic to the function space ''D'' → ''D'', of functions on itself. However, no nontrivial such ''D'' can exist, by [[cardinality]] constraints because the set of all functions from ''D'' into ''D'' has greater cardinality than ''D''.
 
In the 1970s, [[Dana Scott]] showed that, if only [[Scott continuity|continuous functions]] were considered, a set or [[Domain theory|domain]] ''D'' with the required property could be found, thus providing a [[Model theory|model]] for the lambda calculus.
 
This work also formed the basis for the [[denotational semantics]] of programming languages.
 
==See also==
<div style="-moz-column-count:2; column-count:2;">
* [[Applicative computing systems]] – Treatment of [[object (computer science)|object]]s in the style of the lambda calculus
* [[Binary lambda calculus]] – A version of lambda calculus with binary I/O, a binary encoding of terms, and a designated universal machine.
* [[Calculus of constructions]] – A typed lambda calculus with [[type system|type]]s as first-class values
* [[Cartesian closed category]] – A setting for lambda calculus in [[category theory]]
* [[Categorical abstract machine]] – A [[model of computation]] applicable to lambda calculus
* [[Combinatory logic]] – A notation for [[mathematical logic]] without variables
* [[Curry&ndash;Howard isomorphism]] – The formal correspondence between programs and [[mathematical proof|proof]]s
* [[Domain theory]] – Study of certain [[partially ordered sets|posets]] giving [[denotational semantics]] for lambda calculus
* [[Evaluation strategy]] – Rules for the evaluation of expressions in [[programming language]]s
* [[Explicit substitution]] – The theory of substitution, as used in [[#β-reduction|β-reduction]]
* [[Harrop formula]] – A kind of constructive logical formula such that proofs are lambda terms
* [[Kappa calculus]] – A first-order analogue of lambda calculus
* [[Kleene&ndash;Rosser paradox]] – A demonstration that some form of lambda calculus is inconsistent
* [[Knights of the Lambda Calculus]] – A semi-fictional organization of [[Lisp programming language|LISP]] and [[Scheme (programming language)|Scheme]] [[Hacker (programmer subculture)|hacker]]s
* [[Lambda cube]] – A framework for some extensions of typed lambda calculus
* [[Lambda-mu calculus]] – An extension of the lambda calculus for treating [[classical logic]]
* [[Rewriting]] – Transformation of formulæ in formal systems
* [[SECD machine]] – A [[virtual machine]] designed for the lambda calculus
* [[Simply typed lambda calculus]] - Version(s) with a single type constructor
* [[SKI combinator calculus]] – A computational system based on the '''[[#S|S]]''', '''[[#K|K]]''' and '''[[#I|I]]''' combinators
* [[System F]] – A typed lambda calculus with [[type system|type]]-variables
* [[Typed lambda calculus]] – Lambda calculus with [[type system|typed]] variables (and functions)
* [[Universal Turing machine]] – A formal computing machine that is equivalent to lambda calculus
* [[Unlambda]] – An [[esoteric programming language|esoteric]] [[functional programming language|functional]] [[programming language]] based on combinatory logic
</div>
 
==References==
{{Reflist}}
 
==Further reading==
*Abelson, Harold & Gerald Jay Sussman. [[Structure and Interpretation of Computer Programs]]. [[The MIT Press]]. ISBN 0-262-51087-1.
*Hendrik Pieter Barendregt [ftp://ftp.cs.ru.nl/pub/CompMath.Found/lambda.pdf ''Introduction to Lambda Calculus''].
*Henk Barendregt, [http://people.emich.edu/pstephen/other_papers/Impact%20of%20the%20Lambda%20Calculus.pdf The Impact of the Lambda Calculus in Logic and Computer Science]{{Dead link|date=August 2013}}. The Bulletin of Symbolic Logic, Volume 3, Number 2, June 1997.
*[[Hendrik Pieter Barendregt|Barendregt, Hendrik Pieter]], ''The Type Free Lambda Calculus'' pp1091–1132 of ''Handbook of Mathematical Logic'', [[North-Holland]] (1977) ISBN 0-7204-2285-X
*Cardone and Hindley, 2006. [http://www-maths.swan.ac.uk/staff/jrh/papers/JRHHislamWeb.pdf History of Lambda-calculus and Combinatory Logic]{{Dead link|date=July 2012}}. In Gabbay and Woods (eds.), ''Handbook of the History of Logic'', vol. 5. Elsevier.
*Church, Alonzo, ''An unsolvable problem of elementary number theory'', [[American Journal of Mathematics]], 58 (1936), pp.&nbsp;345&ndash;363. This paper contains the proof that the equivalence of lambda expressions is in general not decidable.
*Kleene, Stephen, ''A theory of positive integers in formal logic'', [[American Journal of Mathematics]], 57 (1935), pp.&nbsp;153&ndash;173 and 219&ndash;244. Contains the lambda calculus definitions of several familiar functions.
*[[Peter Landin|Landin, Peter]], ''A Correspondence Between ALGOL 60 and Church's Lambda-Notation'', [[Communications of the ACM]], vol. 8, no. 2 (1965), pages 89–101. Available from the [http://portal.acm.org/citation.cfm?id=363749&coll=portal&dl=ACM ACM site]. A classic paper highlighting the importance of lambda calculus as a basis for programming languages.
*Larson, Jim, [http://www.jetcafe.org/~jim/lambda.html ''An Introduction to Lambda Calculus and Scheme'']. A gentle introduction for programmers.
*Schalk, A. and Simmons, H. (2005) ''[http://www.cs.man.ac.uk/~hsimmons/BOOKS/lcalculus.pdf An introduction to λ-calculi and arithmetic with a decent selection of exercises]. Notes for a course in the Mathematical Logic MSc at Manchester University.
*de Queiroz, Ruy J.G.B. (2008) [http://www.springerlink.com/content/27nk266126k817gq/ ''On Reduction Rules, Meaning-as-Use and Proof-Theoretic Semantics'']. [[Studia Logica]], 90(2):211-247. A paper giving a formal underpinning to the idea of 'meaning-is-use' which, even if based on proofs, it is different from proof-theoretic semantics as in the Dummett–Prawitz tradition since it takes reduction as the rules giving meaning.
Monographs/textbooks for graduate students:
* Morten Heine Sørensen, Paweł Urzyczyn, ''Lectures on the Curry-Howard isomorphism'', Elsevier, 2006, ISBN 0-444-52077-5 is a recent monograph that covers the main topics of lambda calculus from the type-free variety, to most [[typed lambda calculi]], including more recent developments like [[pure type system]]s and the [[lambda cube]]. It does not cover [[subtyping]] extensions.
* {{Citation|last=Pierce|first=Benjamin|title=Types and Programming Languages|publisher=MIT Press|year=2002|isbn=0-262-16209-1}} covers lambda calculi from a practical [[type system]] perspective; some topics like dependent types are only mentioned, but subtyping is an important topic.
 
''Some parts of this article are based on material from [[Free On-line Dictionary of Computing|FOLDOC]], used with [[Wikipedia:Foldoc license|permission]].''
 
==External links==
* {{springer|title=Lambda-calculus|id=p/l057000}}
*Achim Jung, ''[http://www.cs.bham.ac.uk/~axj/pub/papers/lambda-calculus.pdf A Short Introduction to the Lambda Calculus]''-([[Portable Document Format|PDF]])
*Dana Scott, ''[http://turing100.acm.org/lambda_calculus_timeline.pdf A timeline of lambda calculus]''-([[Portable Document Format|PDF]])
*David C. Keenan, ''[http://dkeenan.com/Lambda/ To Dissect a Mockingbird: A Graphical Notation for the Lambda Calculus with Animated Reduction]''
*Raúl Rojas, ''[http://www.inf.fu-berlin.de/lehre/WS03/alpi/lambda.pdf A Tutorial Introduction to the Lambda Calculus]''-([[Portable Document Format|PDF]])
* Peter Selinger, ''[http://www.mscs.dal.ca/~selinger/papers/#lambdanotes Lecture Notes on the Lambda Calculus]''-([[Portable Document Format|PDF]])
*L. Allison, ''[http://www.allisons.org/ll/FP/Lambda/Examples/ Some executable λ-calculus examples]''
*Georg P. Loczewski, [http://www.lambda-bound.com/book/lambdacalc/lcalconl.html ''The Lambda Calculus and A++'']
* Bret Victor, ''[http://worrydream.com/AlligatorEggs/ Alligator Eggs: A Puzzle Game Based on Lambda Calculus]''
*''[http://www.safalra.com/science/lambda-calculus/ Lambda Calculus]'' on [http://www.safalra.com/ Safalra’s Website]
*''{{planetmath reference|id=2788|title=Lambda Calculus}}''
* [http://lci.sourceforge.net/ LCI Lambda Interpreter] a simple yet powerful pure calculus interpreter
* [http://lambda-the-ultimate.org/classic/lc.html Lambda Calculus links on Lambda-the-Ultimate]
*Mike Thyer, [http://thyer.name/lambda-animator/ Lambda Animator], a graphical Java applet demonstrating alternative reduction strategies.
* [http://www.jetcafe.org/~jim/lambda.html An Introduction to Lambda Calculus and Scheme], by Jim Larson
* [http://matt.might.net/articles/c++-template-meta-programming-with-lambda-calculus/ Implementing the Lambda calculus] using [[C++ Templates]]
* Marius Buliga, [http://imar.ro/~mbuliga/graphic_revised.pdf ''Graphic lambda calculus'']
* [http://cs.adelaide.edu.au/~pmk/publications/wage2008.pdf ''Lambda Calculus as a Workflow Model''] by Peter Kelly, Paul Coddington, and Andrew Wendelborn; mentions [[graph reduction]] as a common means of evaluating lambda expressions and discusses the applicability of lambda calculus for [[distributed computing]] (due to the [[Church–Rosser theorem|Church–Rosser]] property, which enables [[parallel computing|parallel]] graph reduction for lambda expressions).
 
 
{{DEFAULTSORT:Lambda Calculus}}
[[Category:1936 in computer science]]
[[Category:American inventions]]
[[Category:Articles with example code]]
[[Category:Computability theory]]
[[Category:Formal methods]]
[[Category:Lambda calculus| ]]
[[Category:Models of computation]]
[[Category:Theoretical computer science]]

Latest revision as of 12:44, 23 December 2014

Greetings. The author's name is Kourtney but she doesn't like when people use her full identity. Her husband doesn't so comprehensive the way she does but what she really likes doing is jogging and she'll be starting something else along with it. He works as a payroll sales person. Vermont is lifting place I've been residing in and Vehicles every day living at this site. Go to my web site find out more: http://dcfm.ca/xe/index.php?mid=news&listStyle=webzine&document_srl=1041097

My web-site :: nicki minaj and lil wayne sex tape online