Documentation

Mathlib.CategoryTheory.Preadditive.Schur

Schur's lemma #

We first prove the part of Schur's Lemma that holds in any preadditive category with kernels, that any nonzero morphism between simple objects is an isomorphism.

Second, we prove Schur's lemma for 𝕜-linear categories with finite dimensional hom spaces, over an algebraically closed field 𝕜: the hom space X ⟶ Y between simple objects X and Y is at most one dimensional, and is 1-dimensional iff X and Y are isomorphic.

The part of Schur's lemma that holds in any preadditive category with kernels: that a nonzero morphism between simple objects is an isomorphism.

As a corollary of Schur's lemma for preadditive categories, any morphism between simple objects is (exclusively) either an isomorphism or zero.

In any preadditive category with kernels, the endomorphisms of a simple object form a division ring.

Equations
  • One or more equations did not get rendered due to their size.

Part of Schur's lemma for 𝕜-linear categories: the hom space between two non-isomorphic simple objects is 0-dimensional.

theorem CategoryTheory.finrank_endomorphism_eq_one {C : Type u_1} [CategoryTheory.Category.{u_3, u_1} C] [CategoryTheory.Preadditive C] (𝕜 : Type u_2) [Field 𝕜] [IsAlgClosed 𝕜] [CategoryTheory.Linear 𝕜 C] {X : C} (isIso_iff_nonzero : ∀ (f : X X), CategoryTheory.IsIso f f 0) [I : FiniteDimensional 𝕜 (X X)] :

An auxiliary lemma for Schur's lemma.

If X ⟶ X is finite dimensional, and every nonzero endomorphism is invertible, then X ⟶ X is 1-dimensional.

Schur's lemma for endomorphisms in 𝕜-linear categories.

Endomorphisms of a simple object form a field if they are finite dimensional. This can't be an instance as 𝕜 would be undetermined.

Equations
Instances For

    Schur's lemma for 𝕜-linear categories: if hom spaces are finite dimensional, then the hom space between simples is at most 1-dimensional.

    See finrank_hom_simple_simple_eq_one_iff and finrank_hom_simple_simple_eq_zero_iff below for the refinements when we know whether or not the simples are isomorphic.