Documentation

ConNF.FOA.FlexApprox

Flexible approximations #

In this file, we define flexible approximations.

Main declarations #

TODO: Fix definition in blueprint to this.

Instances For
    theorem ConNF.BaseAction.FlexApprox.mono [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {A : β } {ξ ζ : BaseAction} {ψ : BaseApprox} ( : FlexApprox A ξ ψ) (h : ζ ξ) :
    FlexApprox A ζ ψ
    theorem ConNF.BaseAction.smul_nearLitter_of_smul_litter [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {ξ : BaseAction} {ψ : BaseApprox} {A : β } {π : BasePerm} {N₁ N₂ : NearLitter} ( : FlexApprox A ξ ψ) ( : ψ.ExactlyApproximates π) (hNξ : ξ N₁ N₂) (hNπ : π N₁ = N₂) :
    π N₁ = N₂

    The main lemma about how approximations interact with actions.

    Equations
    Instances For

      TODO: Move this to PermutativeExtension and do it abstractly.

      Equations
      Instances For
        theorem ConNF.BaseAction.litterPerm_eq [Params] {ξ : BaseAction} {L₁ L₂ : Litter} (h : ξ L₁ L₂) :
        ξ.litterPerm L₁ = L₂
        Equations
        Instances For
          Equations
          Instances For
            theorem ConNF.BaseAction.litter_of_atomPerm [Params] {ξ : BaseAction} {a₁ a₂ : Atom} :
            ξ.atomPerm a₁ a₂ξ a₁ a₂ a₁ξ.dom a₂ξ.codom a₂ = ξ.litterPerm a₁
            theorem ConNF.BaseAction.atomPerm_mem_iff_mem [Params] {ξ : BaseAction} ( : ξ.Nice) {a₁ a₂ : Atom} {N₁ N₂ : NearLitter} (ha : ξ.atomPerm a₁ a₂) (hN : ξ N₁ N₂) :
            a₁ N₁ a₂ N₂
            theorem ConNF.BaseAction.atomPerm_mem_iff [Params] {ξ : BaseAction} ( : ξ.Nice) {N₁ N₂ : NearLitter} (hN : ξ N₁ N₂) (a₂ : Atom) :
            a₂ N₂ (∃ a₁N₁, ξ.atomPerm a₁ a₂) a₂ξ.atomPerm.dom a₂ = N₂
            Equations
            Instances For
              Equations
              Instances For
                Equations
                Instances For
                  theorem ConNF.BaseAction.flexApprox_flexApprox' [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {ξ : BaseAction} {A : β } (hξ₁ : ξ.MapFlexible A) (hξ₂ : ξ.Nice) :

                  A flexible approximation for ξ along A.

                  Equations
                  Instances For