Menu
Home Explore People Places Arts History Plants & Animals Science Life & Culture Technology
On this page
Bijection, injection and surjection
Properties of mathematical functions
surjectivenon-surjective
injective

bijective

injective-only

non-

injective

surjective-only

general

In mathematics, injections, surjections, and bijections are classes of functions distinguished by the manner in which arguments (input expressions from the domain) and images (output expressions from the codomain) are related or mapped to each other.

A function maps elements from its domain to elements in its codomain. Given a function f : X → Y {\displaystyle f\colon X\to Y} :

  • The function is injective, or one-to-one, if each element of the codomain is mapped to by at most one element of the domain, or equivalently, if distinct elements of the domain map to distinct elements in the codomain. An injective function is also called an injection. Notationally:
∀ x , x ′ ∈ X , f ( x ) = f ( x ′ ) ⟹ x = x ′ , {\displaystyle \forall x,x'\in X,f(x)=f(x')\implies x=x',} or, equivalently (using logical transposition), ∀ x , x ′ ∈ X , x ≠ x ′ ⟹ f ( x ) ≠ f ( x ′ ) . {\displaystyle \forall x,x'\in X,x\neq x'\implies f(x)\neq f(x').} 234
  • The function is surjective, or onto, if each element of the codomain is mapped to by at least one element of the domain; that is, if the image and the codomain of the function are equal. A surjective function is a surjection. Notationally:
∀ y ∈ Y , ∃ x ∈ X , y = f ( x ) . {\displaystyle \forall y\in Y,\exists x\in X,y=f(x).} 678
  • The function is bijective (one-to-one and onto, one-to-one correspondence, or invertible) if each element of the codomain is mapped to by exactly one element of the domain; that is, if the function is both injective and surjective. A bijective function is also called a bijection. That is, combining the definitions of injective and surjective,
∀ y ∈ Y , ∃ ! x ∈ X , y = f ( x ) , {\displaystyle \forall y\in Y,\exists !x\in X,y=f(x),} where ∃ ! x {\displaystyle \exists !x} means "there exists exactly one x".
  • In any case (for any function), the following holds:
∀ x ∈ X , ∃ ! y ∈ Y , y = f ( x ) . {\displaystyle \forall x\in X,\exists !y\in Y,y=f(x).}

An injective function need not be surjective (not all elements of the codomain may be associated with arguments), and a surjective function need not be injective (some images may be associated with more than one argument). The four possible combinations of injective and surjective features are illustrated in the adjacent diagrams.

Related Image Collections Add Image
We don't have any YouTube videos related to Bijection, injection and surjection yet.
We don't have any PDF documents related to Bijection, injection and surjection yet.
We don't have any Books related to Bijection, injection and surjection yet.
We don't have any archived web articles related to Bijection, injection and surjection yet.

Injection

Main article: Injective function

Further information on notation: Function (mathematics) § Notation

A function is injective (one-to-one) if each possible element of the codomain is mapped to by at most one argument. Equivalently, a function is injective if it maps distinct arguments to distinct images. An injective function is an injection.13 The formal definition is the following.

The function f : X → Y {\displaystyle f\colon X\to Y} is injective, if for all x , x ′ ∈ X {\displaystyle x,x'\in X} , f ( x ) = f ( x ′ ) ⇒ x = x ′ . {\displaystyle f(x)=f(x')\Rightarrow x=x'.} 141516

The following are some facts related to injections:

  • A function f : X → Y {\displaystyle f\colon X\to Y} is injective if and only if X {\displaystyle X} is empty or f {\displaystyle f} is left-invertible; that is, there is a function g : f ( X ) → X {\displaystyle g\colon f(X)\to X} such that g ∘ f = {\displaystyle g\circ f=} identity function on X. Here, f ( X ) {\displaystyle f(X)} is the image of f {\displaystyle f} .
  • Since every function is surjective when its codomain is restricted to its image, every injection induces a bijection onto its image. More precisely, every injection f : X → Y {\displaystyle f\colon X\to Y} can be factored as a bijection followed by an inclusion as follows. Let f R : X → f ( X ) {\displaystyle f_{R}\colon X\rightarrow f(X)} be f {\displaystyle f} with codomain restricted to its image, and let i : f ( X ) → Y {\displaystyle i\colon f(X)\to Y} be the inclusion map from f ( X ) {\displaystyle f(X)} into Y {\displaystyle Y} . Then f = i ∘ f R {\displaystyle f=i\circ f_{R}} . A dual factorization is given for surjections below.
  • The composition of two injections is again an injection, but if g ∘ f {\displaystyle g\circ f} is injective, then it can only be concluded that f {\displaystyle f} is injective (see figure).
  • Every embedding is injective.

Surjection

Main article: Surjective function

A function is surjective or onto if each element of the codomain is mapped to by at least one element of the domain. In other words, each element of the codomain has a non-empty preimage. Equivalently, a function is surjective if its image is equal to its codomain. A surjective function is a surjection.17 The formal definition is the following.

The function f : X → Y {\displaystyle f\colon X\to Y} is surjective, if for all y ∈ Y {\displaystyle y\in Y} , there is x ∈ X {\displaystyle x\in X} such that f ( x ) = y . {\displaystyle f(x)=y.} 181920

The following are some facts related to surjections:

  • A function f : X → Y {\displaystyle f\colon X\to Y} is surjective if and only if it is right-invertible; that is, if and only if there is a function g : Y → X {\displaystyle g\colon Y\to X} such that f ∘ g = {\displaystyle f\circ g=} identity function on Y {\displaystyle Y} . (This statement is equivalent to the axiom of choice.)
  • By collapsing all arguments mapping to a given fixed image, every surjection induces a bijection from a quotient set of its domain to its codomain. More precisely, the preimages under f of the elements of the image of f {\displaystyle f} are the equivalence classes of an equivalence relation on the domain of f {\displaystyle f} , such that x and y are equivalent if and only they have the same image under f {\displaystyle f} . As all elements of any one of these equivalence classes are mapped by f {\displaystyle f} on the same element of the codomain, this induces a bijection between the quotient set by this equivalence relation (the set of the equivalence classes) and the image of f {\displaystyle f} (which is its codomain when f {\displaystyle f} is surjective). Moreover, f is the composition of the canonical projection from f to the quotient set, and the bijection between the quotient set and the codomain of f {\displaystyle f} .
  • The composition of two surjections is again a surjection, but if g ∘ f {\displaystyle g\circ f} is surjective, then it can only be concluded that g {\displaystyle g} is surjective (see figure).

Bijection

Main article: Bijective function

A function is bijective if it is both injective and surjective. A bijective function is also called a bijection or a one-to-one correspondence (not to be confused with one-to-one function, which refers to injection). A function is bijective if and only if every possible image is mapped to by exactly one argument.21 This equivalent condition is formally expressed as follows:

The function f : X → Y {\displaystyle f\colon X\to Y} is bijective, if for all y ∈ Y {\displaystyle y\in Y} , there is a unique x ∈ X {\displaystyle x\in X} such that f ( x ) = y . {\displaystyle f(x)=y.} 222324

The following are some facts related to bijections:

  • A function f : X → Y {\displaystyle f\colon X\to Y} is bijective if and only if it is invertible; that is, there is a function g : Y → X {\displaystyle g\colon Y\to X} such that g ∘ f = {\displaystyle g\circ f=} identity function on X {\displaystyle X} and f ∘ g = {\displaystyle f\circ g=} identity function on Y {\displaystyle Y} . This function maps each image to its unique preimage.
  • The composition of two bijections is again a bijection, but if g ∘ f {\displaystyle g\circ f} is a bijection, then it can only be concluded that f {\displaystyle f} is injective and g {\displaystyle g} is surjective (see the figure at right and the remarks above regarding injections and surjections).
  • The bijections from a set to itself form a group under composition, called the symmetric group.

Cardinality

Suppose that one wants to define what it means for two sets to "have the same number of elements". One way to do this is to say that two sets "have the same number of elements", if and only if all the elements of one set can be paired with the elements of the other, in such a way that each element is paired with exactly one element. Accordingly, one can define two sets to "have the same number of elements"—if there is a bijection between them. In which case, the two sets are said to have the same cardinality.

Likewise, one can say that set X {\displaystyle X} "has fewer than or the same number of elements" as set Y {\displaystyle Y} , if there is an injection from X {\displaystyle X} to Y {\displaystyle Y} ; one can also say that set X {\displaystyle X} "has fewer than the number of elements" in set Y {\displaystyle Y} , if there is an injection from X {\displaystyle X} to Y {\displaystyle Y} , but not a bijection between X {\displaystyle X} and Y {\displaystyle Y} .

Examples

It is important to specify the domain and codomain of each function, since by changing these, functions which appear to be the same may have different properties.

Injective and surjective (bijective)
  • The identity function idX for every non-empty set X, and thus specifically R → R : x ↦ x . {\displaystyle \mathbf {R} \to \mathbf {R} :x\mapsto x.}
  • R + → R + : x ↦ x 2 {\displaystyle \mathbf {R} ^{+}\to \mathbf {R} ^{+}:x\mapsto x^{2}} , and thus also its inverse R + → R + : x ↦ x . {\displaystyle \mathbf {R} ^{+}\to \mathbf {R} ^{+}:x\mapsto {\sqrt {x}}.}
  • The exponential function exp : R → R + : x ↦ e x {\displaystyle \exp \colon \mathbf {R} \to \mathbf {R} ^{+}:x\mapsto \mathrm {e} ^{x}} (that is, the exponential function with its codomain restricted to its image), and thus also its inverse the natural logarithm ln : R + → R : x ↦ ln ⁡ x . {\displaystyle \ln \colon \mathbf {R} ^{+}\to \mathbf {R} :x\mapsto \ln {x}.} Here, R + {\displaystyle \mathbf {R} ^{+}} denotes the positive real numbers.
  • R → R : x ↦ x 3 {\displaystyle \mathbf {R} \to \mathbf {R} :x\mapsto x^{3}}
Injective and non-surjective
  • The exponential function exp : R → R : x ↦ e x . {\displaystyle \exp \colon \mathbf {R} \to \mathbf {R} :x\mapsto \mathrm {e} ^{x}.}
Non-injective and surjective
  • R → R : x ↦ ( x − 1 ) x ( x + 1 ) = x 3 − x . {\displaystyle \mathbf {R} \to \mathbf {R} :x\mapsto (x-1)x(x+1)=x^{3}-x.}
  • R → [ − 1 , 1 ] : x ↦ sin ⁡ ( x ) . {\displaystyle \mathbf {R} \to [-1,1]:x\mapsto \sin(x).}
Non-injective and non-surjective
  • R → R : x ↦ sin ⁡ ( x ) . {\displaystyle \mathbf {R} \to \mathbf {R} :x\mapsto \sin(x).}
  • R → R : x ↦ x 2 {\displaystyle \mathbf {R} \to \mathbf {R} :x\mapsto x^{2}}

Properties

  • For every function f, let X be a subset of the domain and Y a subset of the codomain. One has always Xf−1(f(X)) and f(f−1(Y)) ⊆ Y, where f(X) is the image of X and f−1(Y) is the preimage of Y under f. If f is injective, then X = f−1(f(X)), and if f is surjective, then f(f−1(Y)) = Y.
  • For every function h : XY, one can define a surjection H : Xh(X) : xh(x) and an injection I : h(X) → Y : yy. It follows that ⁠ h = I ∘ H {\displaystyle h=I\circ H} ⁠. This decomposition as the composition of a surjection and an injection is unique up to an isomorphism, in the sense that, given such a decomposition, there is a unique bijection φ : h ( X ) → H ( X ) {\displaystyle \varphi :h(X)\to H(X)} such that H ( x ) = φ ( h ( x ) ) {\displaystyle H(x)=\varphi (h(x))} and I ( φ ( h ( x ) ) ) = h ( x ) {\displaystyle I(\varphi (h(x)))=h(x)} for every x ∈ X . {\displaystyle x\in X.}

Category theory

In the category of sets, injections, surjections, and bijections correspond precisely to monomorphisms, epimorphisms, and isomorphisms, respectively.25

History

The Oxford English Dictionary records the use of the word injection as a noun by S. Mac Lane in Bulletin of the American Mathematical Society (1950), and injective as an adjective by Eilenberg and Steenrod in Foundations of Algebraic Topology (1952).26

However, it was not until the French Bourbaki group coined the injective-surjective-bijective terminology (both as nouns and adjectives) that they achieved widespread adoption.27

See also

References

  1. "Injective, Surjective and Bijective". www.mathsisfun.com. Retrieved 2019-12-07. https://www.mathsisfun.com/sets/injective-surjective-bijective.html

  2. "Bijection, Injection, And Surjection | Brilliant Math & Science Wiki". brilliant.org. Retrieved 2019-12-07. https://brilliant.org/wiki/bijection-injection-and-surjection/

  3. Farlow, S. J. "Injections, Surjections, and Bijections" (PDF). math.umaine.edu. Archived from the original (PDF) on 2020-01-10. Retrieved 2019-12-06. /wiki/Stanley_Farlow

  4. "6.3: Injections, Surjections, and Bijections". Mathematics LibreTexts. 2017-09-20. Retrieved 2019-12-07. https://math.libretexts.org/Bookshelves/Mathematical_Logic_and_Proof/Book%3A_Mathematical_Reasoning_-_Writing_and_Proof_(Sundstrom)/6%3A_Functions/6.3%3A_Injections%2C_Surjections%2C_and_Bijections

  5. "Injective, Surjective and Bijective". www.mathsisfun.com. Retrieved 2019-12-07. https://www.mathsisfun.com/sets/injective-surjective-bijective.html

  6. "Bijection, Injection, And Surjection | Brilliant Math & Science Wiki". brilliant.org. Retrieved 2019-12-07. https://brilliant.org/wiki/bijection-injection-and-surjection/

  7. Farlow, S. J. "Injections, Surjections, and Bijections" (PDF). math.umaine.edu. Archived from the original (PDF) on 2020-01-10. Retrieved 2019-12-06. /wiki/Stanley_Farlow

  8. "6.3: Injections, Surjections, and Bijections". Mathematics LibreTexts. 2017-09-20. Retrieved 2019-12-07. https://math.libretexts.org/Bookshelves/Mathematical_Logic_and_Proof/Book%3A_Mathematical_Reasoning_-_Writing_and_Proof_(Sundstrom)/6%3A_Functions/6.3%3A_Injections%2C_Surjections%2C_and_Bijections

  9. "Injective, Surjective and Bijective". www.mathsisfun.com. Retrieved 2019-12-07. https://www.mathsisfun.com/sets/injective-surjective-bijective.html

  10. "Bijection, Injection, And Surjection | Brilliant Math & Science Wiki". brilliant.org. Retrieved 2019-12-07. https://brilliant.org/wiki/bijection-injection-and-surjection/

  11. Farlow, S. J. "Injections, Surjections, and Bijections" (PDF). math.umaine.edu. Archived from the original (PDF) on 2020-01-10. Retrieved 2019-12-06. /wiki/Stanley_Farlow

  12. "6.3: Injections, Surjections, and Bijections". Mathematics LibreTexts. 2017-09-20. Retrieved 2019-12-07. https://math.libretexts.org/Bookshelves/Mathematical_Logic_and_Proof/Book%3A_Mathematical_Reasoning_-_Writing_and_Proof_(Sundstrom)/6%3A_Functions/6.3%3A_Injections%2C_Surjections%2C_and_Bijections

  13. "Injective, Surjective and Bijective". www.mathsisfun.com. Retrieved 2019-12-07. https://www.mathsisfun.com/sets/injective-surjective-bijective.html

  14. "Bijection, Injection, And Surjection | Brilliant Math & Science Wiki". brilliant.org. Retrieved 2019-12-07. https://brilliant.org/wiki/bijection-injection-and-surjection/

  15. Farlow, S. J. "Injections, Surjections, and Bijections" (PDF). math.umaine.edu. Archived from the original (PDF) on 2020-01-10. Retrieved 2019-12-06. /wiki/Stanley_Farlow

  16. "6.3: Injections, Surjections, and Bijections". Mathematics LibreTexts. 2017-09-20. Retrieved 2019-12-07. https://math.libretexts.org/Bookshelves/Mathematical_Logic_and_Proof/Book%3A_Mathematical_Reasoning_-_Writing_and_Proof_(Sundstrom)/6%3A_Functions/6.3%3A_Injections%2C_Surjections%2C_and_Bijections

  17. "Injective, Surjective and Bijective". www.mathsisfun.com. Retrieved 2019-12-07. https://www.mathsisfun.com/sets/injective-surjective-bijective.html

  18. "Bijection, Injection, And Surjection | Brilliant Math & Science Wiki". brilliant.org. Retrieved 2019-12-07. https://brilliant.org/wiki/bijection-injection-and-surjection/

  19. Farlow, S. J. "Injections, Surjections, and Bijections" (PDF). math.umaine.edu. Archived from the original (PDF) on 2020-01-10. Retrieved 2019-12-06. /wiki/Stanley_Farlow

  20. "6.3: Injections, Surjections, and Bijections". Mathematics LibreTexts. 2017-09-20. Retrieved 2019-12-07. https://math.libretexts.org/Bookshelves/Mathematical_Logic_and_Proof/Book%3A_Mathematical_Reasoning_-_Writing_and_Proof_(Sundstrom)/6%3A_Functions/6.3%3A_Injections%2C_Surjections%2C_and_Bijections

  21. "Injective, Surjective and Bijective". www.mathsisfun.com. Retrieved 2019-12-07. https://www.mathsisfun.com/sets/injective-surjective-bijective.html

  22. "Bijection, Injection, And Surjection | Brilliant Math & Science Wiki". brilliant.org. Retrieved 2019-12-07. https://brilliant.org/wiki/bijection-injection-and-surjection/

  23. Farlow, S. J. "Injections, Surjections, and Bijections" (PDF). math.umaine.edu. Archived from the original (PDF) on 2020-01-10. Retrieved 2019-12-06. /wiki/Stanley_Farlow

  24. "6.3: Injections, Surjections, and Bijections". Mathematics LibreTexts. 2017-09-20. Retrieved 2019-12-07. https://math.libretexts.org/Bookshelves/Mathematical_Logic_and_Proof/Book%3A_Mathematical_Reasoning_-_Writing_and_Proof_(Sundstrom)/6%3A_Functions/6.3%3A_Injections%2C_Surjections%2C_and_Bijections

  25. "Section 7.3 (00V5): Injective and surjective maps of presheaves—The Stacks project". stacks.math.columbia.edu. Retrieved 2019-12-07. https://stacks.math.columbia.edu/tag/00V5

  26. "Earliest Known Uses of Some of the Words of Mathematics (I)". jeff560.tripod.com. Retrieved 2022-06-11. https://jeff560.tripod.com/i.html

  27. Mashaal, Maurice (2006). Bourbaki. American Mathematical Soc. p. 106. ISBN 978-0-8218-3967-6. 978-0-8218-3967-6