Documentation

ConNF.FOA.StrAction

Structural actions #

In this file, we define structural actions, and prove the freedom of action theorem for actions.

Main declarations #

@[reducible, inline]
Equations
Instances For
    Equations
    Instances For
      theorem ConNF.StrAction.Coherent.deriv [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {ξ : StrAction β} ( : ξ.Coherent) {γ : TypeIndex} [LeLevel γ] (A : β γ) :
      Coherent (ξ A)

      TODO: Maybe move this to BaseActionClass?

      • atoms (a₁ a₂ : Atom) : ξ a₁ a₂a₂ = π a₁
      • nearLitters (N₁ N₂ : NearLitter) : ξ N₁ N₂N₂ = π N₁
      Instances For
        theorem ConNF.BaseAction.Approximates.litters [Params] {ξ : BaseAction} {π : BasePerm} (h : ξ.Approximates π) (L₁ L₂ : Litter) :
        ξ L₁ L₂π L₁ = L₂
        theorem ConNF.BaseAction.Approximates.mono [Params] {ψ χ : BaseAction} {π : BasePerm} ( : χ.Approximates π) (h : ψ χ) :
        Equations
        Instances For
          Equations
          Instances For
            theorem ConNF.StrAction.flexApprox_coherent [Params] [Level] {β : TypeIndex} [LeLevel β] [CoherentData] (ξ : StrAction β) ( : ∀ (A : β ), (ξ A).MapFlexible A) :

            TODO: Put this in the blueprint.