Documentation

Mathlib.CategoryTheory.Subobject.NoetherianObject

Noetherian objects #

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

Future works #

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

Equations
Instances For
    @[reducible, inline]

    An object X in a category C is Noetherian if Subobject X satisfies the ascending chain condition.

    Equations
    Instances For
      theorem CategoryTheory.isNoetherianObject_iff_monotone_chain_condition {C : Type u} [Category.{v, u} C] (X : C) :
      IsNoetherianObject X ∀ (f : →o Subobject X), ∃ (n : ), ∀ (m : ), n mf n = f m
      theorem CategoryTheory.monotone_chain_condition_of_isNoetherianObject {C : Type u} [Category.{v, u} C] {X : C} [IsNoetherianObject X] (f : →o Subobject X) :
      ∃ (n : ), ∀ (m : ), n mf n = f m