Documentation

Mathlib.CategoryTheory.Subobject.ArtinianObject

Artinian objects #

We shall say that an object X in a category C is Artinian (type class IsArtinianObject X) if the ordered type Subobject X satisfies the descending chain condition. The corresponding property of objects isArtinianObject : ObjectProperty C is always closed under subobjects.

Future works #

An object X in a category C is Artinian if Subobject X satisfies the descending chain condition. This definition is a term in ObjectProperty C which allows to study the stability properties of Artinian objects. For statements regarding specific objects, it is advisable to use the type class IsArtinianObject instead.

Stacks Tag 0FCF

Equations
Instances For
    @[reducible, inline]

    An object X in a category C is Artinian if Subobject X satisfies the descending chain condition.

    Stacks Tag 0FCF

    Equations
    Instances For
      theorem CategoryTheory.isArtinianObject_iff_antitone_chain_condition {C : Type u} [Category.{v, u} C] (X : C) :
      IsArtinianObject X ∀ (f : →o (Subobject X)ᵒᵈ), ∃ (n : ), ∀ (m : ), n mf n = f m
      theorem CategoryTheory.antitone_chain_condition_of_isArtinianObject {C : Type u} [Category.{v, u} C] {X : C} [IsArtinianObject X] (f : →o (Subobject X)ᵒᵈ) :
      ∃ (n : ), ∀ (m : ), n mf n = f m

      Choose an arbitrary simple subobject of a non-zero Artinian object.

      Equations
      Instances For

        The monomorphism from the arbitrary simple subobject of a non-zero artinian object.

        Equations
        Instances For