Documentation

ConNF.FOA.LAction.StructLAction

Structural litter actions #

In this file, we define structural litter actions, which are trees of base litter actions.

Main declarations #

@[reducible, inline]
abbrev ConNF.StructLAction [ConNF.Params] (α : ConNF.TypeIndex) :

A β-structural action is a β-tree of base litter actions.

Equations
Instances For
    def ConNF.StructLAction.Lawful [ConNF.Params] {β : ConNF.TypeIndex} (φ : ConNF.StructLAction β) :
    Equations
    Instances For
      Equations
      Instances For
        def ConNF.StructLAction.MapFlexible [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.FOAAssumptions] {β : ConNF.Λ} (φ : ConNF.StructLAction β) :

        This structural action maps flexible litters to flexible litters.

        Equations
        Instances For
          def ConNF.StructLAction.Precise [ConNF.Params] {β : ConNF.TypeIndex} (φ : ConNF.StructLAction β) :
          Equations
          Instances For
            noncomputable def ConNF.StructLAction.complete [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.FOAAssumptions] {β : ConNF.Λ} (φ : ConNF.StructLAction β) (hφ : φ.Lawful) :
            Equations
            • φ.complete B = (φ B).complete B
            Instances For
              theorem ConNF.StructLAction.complete_apply [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.FOAAssumptions] {β : ConNF.Λ} (φ : ConNF.StructLAction β) (hφ : φ.Lawful) (B : ConNF.ExtendedIndex β) :
              φ.complete B = (φ B).complete B
              theorem ConNF.StructLAction.smul_atom_eq [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.FOAAssumptions] {β : ConNF.Λ} (φ : ConNF.StructLAction β) {hφ : φ.Lawful} {π : ConNF.StructPerm β} (hπ : (φ.complete ).ExactlyApproximates π) {a : ConNF.Atom} {B : ConNF.ExtendedIndex β} (ha : ((φ B).atomMap a).Dom) :
              π B a = ((φ B).atomMap a).get ha
              theorem ConNF.StructLAction.smul_toNearLitter_eq_of_precise [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.FOAAssumptions] {β : ConNF.Λ} (φ : ConNF.StructLAction β) {hφ : φ.Lawful} (hφp : φ.Precise) {π : ConNF.StructPerm β} (hπ : (φ.complete ).ExactlyApproximates π) {L : ConNF.Litter} {B : ConNF.ExtendedIndex β} (hL : ((φ B).litterMap L).Dom) (hπL : π B L = (((φ B).litterMap L).get hL).fst) :
              π B L.toNearLitter = ((φ B).litterMap L).get hL
              theorem ConNF.StructLAction.smul_nearLitter_eq_of_precise [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.FOAAssumptions] {β : ConNF.Λ} (φ : ConNF.StructLAction β) {hφ : φ.Lawful} (hφp : φ.Precise) {π : ConNF.StructPerm β} (hπ : (φ.complete ).ExactlyApproximates π) {N : ConNF.NearLitter} {B : ConNF.ExtendedIndex β} (hN : ((φ B).litterMap N.fst).Dom) (hπL : π B N.fst = (((φ B).litterMap N.fst).get hN).fst) :
              (π B N) = symmDiff ((((φ B).litterMap N.fst).get hN)) (ConNF.Tree.comp B π symmDiff (ConNF.litterSet N.fst) N)
              Equations
              theorem ConNF.StructLAction.Lawful.le [ConNF.Params] {β : ConNF.TypeIndex} {φ : ConNF.StructLAction β} {ψ : ConNF.StructLAction β} (h : φ.Lawful) (hψ : ψ φ) :
              ψ.Lawful
              theorem ConNF.StructLAction.le_comp [ConNF.Params] {β : ConNF.TypeIndex} {γ : ConNF.TypeIndex} {φ : ConNF.StructLAction β} {ψ : ConNF.StructLAction β} (h : φ ψ) (A : Quiver.Path β γ) :
              theorem ConNF.StructLAction.Lawful.comp [ConNF.Params] {β : ConNF.TypeIndex} {γ : ConNF.TypeIndex} {φ : ConNF.StructLAction β} (h : φ.Lawful) (A : Quiver.Path β γ) :