mathlib3 documentation

category_theory.preadditive.schur

Schur's lemma #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4. 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.

@[protected, instance]

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

Equations

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

theorem category_theory.finrank_endomorphism_eq_one {C : Type u_1} [category_theory.category C] [category_theory.preadditive C] (π•œ : Type u_3) [field π•œ] [is_alg_closed π•œ] [category_theory.linear π•œ C] {X : C} (is_iso_iff_nonzero : βˆ€ (f : X ⟢ X), category_theory.is_iso f ↔ f β‰  0) [I : finite_dimensional π•œ (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

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.