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]
abbrev ConNF.StrAction [ConNF.Params] :
ConNF.TypeIndexType u
Equations
Instances For
    def ConNF.StrAction.Coherent [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] (ξ : ConNF.StrAction β) :
    Equations
    Instances For
      theorem ConNF.StrAction.Coherent.deriv [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] {ξ : ConNF.StrAction β} (hξ : ξ.Coherent) {γ : ConNF.TypeIndex} [ConNF.LeLevel γ] (A : β γ) :
      theorem ConNF.StrAction.mapFlexible_of_coherent [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] {ξ : ConNF.StrAction β} (hξ : ξ.Coherent) (A : β ) :
      (ξ A).MapFlexible A
      structure ConNF.BaseAction.Approximates [ConNF.Params] (ξ : ConNF.BaseAction) (π : ConNF.BasePerm) :

      TODO: Maybe move this to BaseActionClass?

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

            TODO: Put this in the blueprint.