Английская Википедия:Functor

Материал из Онлайн справочника
Перейти к навигацииПерейти к поиску

Шаблон:Short description Шаблон:About Шаблон:Redirect

In mathematics, specifically category theory, a functor is a mapping between categories. Functors were first considered in algebraic topology, where algebraic objects (such as the fundamental group) are associated to topological spaces, and maps between these algebraic objects are associated to continuous maps between spaces. Nowadays, functors are used throughout modern mathematics to relate various categories. Thus, functors are important in all areas within mathematics to which category theory is applied.

The words category and functor were borrowed by mathematicians from the philosophers Aristotle and Rudolf Carnap, respectively.[1] The latter used functor in a linguistic context;[2] see function word.

Definition

Шаблон:Technical

Файл:Commutative diagram for morphism.svg
A category with objects X, Y, Z and morphisms f, g, g ∘ f
Файл:Commutative diagram of a functor.svg
Functor <math>F</math> must preserve the composition of morphisms <math>g</math> and <math>f</math>

Let C and D be categories. A functor F from C to D is a mapping thatШаблон:Sfnp

  • associates each object <math>X</math> in C to an object <math>F(X)</math> in D,
  • associates each morphism <math>f \colon X \to Y</math> in C to a morphism <math>F(f) \colon F(X) \to F(Y)</math> in D such that the following two conditions hold:
    • <math>F(\mathrm{id}_{X}) = \mathrm{id}_{F(X)}\,\!</math> for every object <math>X</math> in C,
    • <math>F(g \circ f) = F(g) \circ F(f)</math> for all morphisms <math>f \colon X \to Y\,\!</math> and <math>g \colon Y\to Z</math> in C.

That is, functors must preserve identity morphisms and composition of morphisms.

Covariance and contravariance

Шаблон:See also There are many constructions in mathematics that would be functors but for the fact that they "turn morphisms around" and "reverse composition". We then define a contravariant functor F from C to D as a mapping that

  • associates each object <math>X</math> in C with an object <math>F(X)</math> in D,
  • associates each morphism <math>f \colon X\to Y</math> in C with a morphism <math>F(f) \colon F(Y) \to F(X)</math> in D such that the following two conditions hold:
    • <math>F(\mathrm{id}_X) = \mathrm{id}_{F(X)}\,\!</math> for every object <math>X</math> in C,
    • <math>F(g \circ f) = F(f) \circ F(g)</math> for all morphisms <math>f \colon X\to Y</math> and <math>g \colon Y\to Z</math> in C.

Note that contravariant functors reverse the direction of composition.

Ordinary functors are also called covariant functors in order to distinguish them from contravariant ones. Note that one can also define a contravariant functor as a covariant functor on the opposite category <math>C^\mathrm{op}</math>.Шаблон:Sfnp Some authors prefer to write all expressions covariantly. That is, instead of saying <math>F \colon C\to D</math> is a contravariant functor, they simply write <math>F \colon C^{\mathrm{op}} \to D</math> (or sometimes <math>F \colon C \to D^{\mathrm{op}}</math>) and call it a functor.

Contravariant functors are also occasionally called cofunctors.[3]

There is a convention which refers to "vectors"—i.e., vector fields, elements of the space of sections <math>\Gamma(TM)</math> of a tangent bundle <math>TM</math>—as "contravariant" and to "covectors"—i.e., 1-forms, elements of the space of sections <math>\Gamma\mathord\left(T^*M\right)</math> of a cotangent bundle <math>T^*M</math>—as "covariant". This terminology originates in physics, and its rationale has to do with the position of the indices ("upstairs" and "downstairs") in expressions such as <math>{x'}^{\,i} = \Lambda^i_j x^j</math> for <math>\mathbf{x}' = \boldsymbol{\Lambda}\mathbf{x}</math> or <math>\omega'_i = \Lambda^j_i \omega_j</math> for <math>\boldsymbol{\omega}' = \boldsymbol{\omega}\boldsymbol{\Lambda}^\textsf{T}.</math> In this formalism it is observed that the coordinate transformation symbol <math>\Lambda^j_i</math> (representing the matrix <math>\boldsymbol{\Lambda}^\textsf{T}</math>) acts on the "covector coordinates" "in the same way" as on the basis vectors: <math>\mathbf{e}_i = \Lambda^j_i\mathbf{e}_j</math>—whereas it acts "in the opposite way" on the "vector coordinates" (but "in the same way" as on the basis covectors: <math>\mathbf{e}^i = \Lambda^i_j \mathbf{e}^j</math>). This terminology is contrary to the one used in category theory because it is the covectors that have pullbacks in general and are thus contravariant, whereas vectors in general are covariant since they can be pushed forward. See also Covariance and contravariance of vectors.

Opposite functor

Every functor <math>F \colon C\to D</math> induces the opposite functor <math>F^\mathrm{op} \colon C^\mathrm{op}\to D^\mathrm{op}</math>, where <math>C^\mathrm{op}</math> and <math>D^\mathrm{op}</math> are the opposite categories to <math>C</math> and <math>D</math>.[4] By definition, <math>F^\mathrm{op}</math> maps objects and morphisms in the identical way as does <math>F</math>. Since <math>C^\mathrm{op}</math> does not coincide with <math>C</math> as a category, and similarly for <math>D</math>, <math>F^\mathrm{op}</math> is distinguished from <math>F</math>. For example, when composing <math>F \colon C_0\to C_1</math> with <math>G \colon C_1^\mathrm{op}\to C_2</math>, one should use either <math>G\circ F^\mathrm{op}</math> or <math>G^\mathrm{op}\circ F</math>. Note that, following the property of opposite category, <math>\left(F^\mathrm{op}\right)^\mathrm{op} = F</math>.

Bifunctors and multifunctors

A bifunctor (also known as a binary functor) is a functor whose domain is a product category. For example, the Hom functor is of the type Шаблон:Nowrap. It can be seen as a functor in two arguments. The Hom functor is a natural example; it is contravariant in one argument, covariant in the other.

A multifunctor is a generalization of the functor concept to n variables. So, for example, a bifunctor is a multifunctor with Шаблон:Nowrap.

Properties

Two important consequences of the functor axioms are:

One can compose functors, i.e. if F is a functor from A to B and G is a functor from B to C then one can form the composite functor Шаблон:Nowrap from A to C. Composition of functors is associative where defined. Identity of composition of functors is the identity functor. This shows that functors can be considered as morphisms in categories of categories, for example in the category of small categories.

A small category with a single object is the same thing as a monoid: the morphisms of a one-object category can be thought of as elements of the monoid, and composition in the category is thought of as the monoid operation. Functors between one-object categories correspond to monoid homomorphisms. So in a sense, functors between arbitrary categories are a kind of generalization of monoid homomorphisms to categories with more than one object.

Examples

Diagram
For categories C and J, a diagram of type J in C is a covariant functor <math>D \colon J\to C</math>.
(Category theoretical) presheaf
For categories C and J, a J-presheaf on C is a contravariant functor <math>D \colon C\to J</math>.Шаблон:ParagraphIn the special case when J is Set, the category of sets and functions, D is called a presheaf on C.
Presheaves (over a topological space)
If X is a topological space, then the open sets in X form a partially ordered set Open(X) under inclusion. Like every partially ordered set, Open(X) forms a small category by adding a single arrow Шаблон:Nowrap if and only if <math>U \subseteq V</math>. Contravariant functors on Open(X) are called presheaves on X. For instance, by assigning to every open set U the associative algebra of real-valued continuous functions on U, one obtains a presheaf of algebras on X.
Constant functor
The functor Шаблон:Nowrap which maps every object of C to a fixed object X in D and every morphism in C to the identity morphism on X. Such a functor is called a constant or selection functor.
Шаблон:TermШаблон:Anchor
A functor that maps a category to that same category; e.g., polynomial functor.
Шаблон:Term
In category C, written 1C or idC, maps an object to itself and a morphism to itself. The identity functor is an endofunctor.
Diagonal functor
The diagonal functor is defined as the functor from D to the functor category DC which sends each object in D to the constant functor at that object.
Limit functor
For a fixed index category J, if every functor Шаблон:Nowrap has a limit (for instance if C is complete), then the limit functor Шаблон:Nowrap assigns to each functor its limit. The existence of this functor can be proved by realizing that it is the right-adjoint to the diagonal functor and invoking the Freyd adjoint functor theorem. This requires a suitable version of the axiom of choice. Similar remarks apply to the colimit functor (which assigns to every functor its colimit, and is covariant).
Power sets functor
The power set functor Шаблон:Nowrap maps each set to its power set and each function <math> f \colon X \to Y</math> to the map which sends <math>U \in \mathcal{P}(X)</math> to its image <math>f(U) \in \mathcal{P}(Y)</math>. One can also consider the contravariant power set functor which sends <math> f \colon X \to Y </math> to the map which sends <math>V \subseteq Y</math> to its inverse image <math>f^{-1}(V) \subseteq X.</math>Шаблон:Paragraph For example, if <math>X = \{0,1\}</math> then <math>F(X) = \mathcal{P}(X) = \{\{\}, \{0\}, \{1\}, X\}</math>. Suppose <math>f(0) = \{\}</math> and <math>f(1) = X</math>. Then <math>F(f)</math> is the function which sends any subset <math>U</math> of <math>X</math> to its image <math>f(U)</math>, which in this case means <math>\{\} \mapsto f(\{\}) = \{\}</math>, where <math>\mapsto</math> denotes the mapping under <math>F(f)</math>, so this could also be written as <math>(F(f))(\{\})= \{\}</math>. For the other values,<math>
   \{0\} \mapsto f(\{0\})   = \{f(0)\}       = \{\{\}\},\ </math> <math>
   \{1\} \mapsto f(\{1\})   = \{f(1)\}       = \{X\},\ </math> <math>
 \{0,1\} \mapsto f(\{0,1\}) = \{f(0), f(1)\} = \{\{\}, X\}.

</math> Note that <math>f(\{0, 1\})</math> consequently generates the trivial topology on <math>X</math>. Also note that although the function <math>f</math> in this example mapped to the power set of <math>X</math>, that need not be the case in general.

Шаблон:Visible anchor
The map which assigns to every vector space its dual space and to every linear map its dual or transpose is a contravariant functor from the category of all vector spaces over a fixed field to itself.
Fundamental group
Consider the category of pointed topological spaces, i.e. topological spaces with distinguished points. The objects are pairs Шаблон:Nowrap, where X is a topological space and x0 is a point in X. A morphism from Шаблон:Nowrap to Шаблон:Nowrap is given by a continuous map Шаблон:Nowrap with Шаблон:Nowrap.Шаблон:Paragraph To every topological space X with distinguished point x0, one can define the fundamental group based at x0, denoted Шаблон:Nowrap. This is the group of homotopy classes of loops based at x0, with the group operation of concatenation. If Шаблон:Nowrap is a morphism of pointed spaces, then every loop in X with base point x0 can be composed with f to yield a loop in Y with base point y0. This operation is compatible with the homotopy equivalence relation and the composition of loops, and we get a group homomorphism from Шаблон:Nowrap to Шаблон:Nowrap. We thus obtain a functor from the category of pointed topological spaces to the category of groups.Шаблон:Paragraph In the category of topological spaces (without distinguished point), one considers homotopy classes of generic curves, but they cannot be composed unless they share an endpoint. Thus one has the fundamental groupoid instead of the fundamental group, and this construction is functorial.
Algebra of continuous functions
A contravariant functor from the category of topological spaces (with continuous maps as morphisms) to the category of real associative algebras is given by assigning to every topological space X the algebra C(X) of all real-valued continuous functions on that space. Every continuous map Шаблон:Nowrap induces an algebra homomorphism Шаблон:Nowrap by the rule Шаблон:Nowrap for every φ in C(Y).
Tangent and cotangent bundles
The map which sends every differentiable manifold to its tangent bundle and every smooth map to its derivative is a covariant functor from the category of differentiable manifolds to the category of vector bundles. Шаблон:ParagraphDoing this constructions pointwise gives the tangent space, a covariant functor from the category of pointed differentiable manifolds to the category of real vector spaces. Likewise, cotangent space is a contravariant functor, essentially the composition of the tangent space with the dual space above.
Group actions/representations
Every group G can be considered as a category with a single object whose morphisms are the elements of G. A functor from G to Set is then nothing but a group action of G on a particular set, i.e. a G-set. Likewise, a functor from G to the category of vector spaces, VectK, is a linear representation of G. In general, a functor Шаблон:Nowrap can be considered as an "action" of G on an object in the category C. If C is a group, then this action is a group homomorphism.
Lie algebras
Assigning to every real (complex) Lie group its real (complex) Lie algebra defines a functor.
Tensor products
If C denotes the category of vector spaces over a fixed field, with linear maps as morphisms, then the tensor product <math>V \otimes W</math> defines a functor Шаблон:Nowrap which is covariant in both arguments.[5]
Forgetful functors
The functor Шаблон:Nowrap which maps a group to its underlying set and a group homomorphism to its underlying function of sets is a functor.Шаблон:Sfnp Functors like these, which "forget" some structure, are termed forgetful functors. Another example is the functor Шаблон:Nowrap which maps a ring to its underlying additive abelian group. Morphisms in Rng (ring homomorphisms) become morphisms in Ab (abelian group homomorphisms).
Free functors
Going in the opposite direction of forgetful functors are free functors. The free functor Шаблон:Nowrap sends every set X to the free group generated by X. Functions get mapped to group homomorphisms between free groups. Free constructions exist for many categories based on structured sets. See free object.
Homomorphism groups
To every pair A, B of abelian groups one can assign the abelian group Hom(A, B) consisting of all group homomorphisms from A to B. This is a functor which is contravariant in the first and covariant in the second argument, i.e. it is a functor Шаблон:Nowrap (where Ab denotes the category of abelian groups with group homomorphisms). If Шаблон:Nowrap and Шаблон:Nowrap are morphisms in Ab, then the group homomorphism Шаблон:Nowrap: Шаблон:Nowrap is given by Шаблон:Nowrap. See Hom functor.
Representable functors
We can generalize the previous example to any category C. To every pair X, Y of objects in C one can assign the set Шаблон:Nowrap of morphisms from X to Y. This defines a functor to Set which is contravariant in the first argument and covariant in the second, i.e. it is a functor Шаблон:Nowrap. If Шаблон:Nowrap and Шаблон:Nowrap are morphisms in C, then the map Шаблон:Nowrap is given by Шаблон:Nowrap.Шаблон:Paragraph Functors like these are called representable functors. An important goal in many settings is to determine whether a given functor is representable.

Relation to other categorical concepts

Let C and D be categories. The collection of all functors from C to D forms the objects of a category: the functor category. Morphisms in this category are natural transformations between functors.

Functors are often defined by universal properties; examples are the tensor product, the direct sum and direct product of groups or vector spaces, construction of free groups and modules, direct and inverse limits. The concepts of limit and colimit generalize several of the above.

Universal constructions often give rise to pairs of adjoint functors.

Computer implementations

Шаблон:Main Functors sometimes appear in functional programming. For instance, the programming language Haskell has a class Functor where fmap is a polytypic function used to map functions (morphisms on Hask, the category of Haskell types)[6] between existing types to functions between some new types.[7]

See also

Шаблон:Portal

Notes

Шаблон:Reflist

References

External links

Шаблон:Wiktionary

Шаблон:Category theory Шаблон:Functors

  1. Шаблон:Citation
  2. Carnap, Rudolf (1937). The Logical Syntax of Language, Routledge & Kegan, pp. 13–14.
  3. Шаблон:Cite book
  4. Шаблон:Citation
  5. Шаблон:Citation
  6. It's not entirely clear that Haskell datatypes truly form a category. See https://wiki.haskell.org/Hask for more details.
  7. See https://wiki.haskell.org/Category_theory/Functor#Functors_in_Haskell for more information.