Documentation

Mathlib.CategoryTheory.Shift.Predicate

Predicates on categories equipped with shift #

Given a predicate P : C → Prop on objects of a category equipped with a shift by A, we define shifted predicates PredicateShift P a for all a : A.

def CategoryTheory.PredicateShift {C : Type u_1} [Category.{u_3, u_1} C] (P : CProp) {A : Type u_2} [AddMonoid A] [HasShift C A] (a : A) :
CProp

Given a predicate P : C → Prop on objects of a category equipped with a shift by A, this is the predicate which is satisfied by X if P (X⟦a⟧).

Equations
Instances For
    theorem CategoryTheory.predicateShift_iff {C : Type u_1} [Category.{u_3, u_1} C] (P : CProp) {A : Type u_2} [AddMonoid A] [HasShift C A] (a : A) (X : C) :
    PredicateShift P a X P ((shiftFunctor C a).obj X)