Documentation

ConNF.Strong.CodingFunction

Coding functions #

In this file, we define coding functions.

Main declarations #

Equations
Instances For
    Equations
    Instances For
      theorem ConNF.Support.orbit_eq_iff [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {S T : Support β} :
      S.orbit = T.orbit ∃ (ρ : AllPerm β), ρ S = T
      @[simp]
      theorem ConNF.Support.smul_orbit [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {S : Support β} {ρ : AllPerm β} :
      (ρ S).orbit = S.orbit
      Instances For
        theorem ConNF.CodingFunction.ext' [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {χ₁ χ₂ : CodingFunction β} (h : ∀ (S : Support β) (x : TSet β), χ₁.rel S x χ₂.rel S x) :
        χ₁ = χ₂
        theorem ConNF.CodingFunction.ext_aux [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {χ₁ χ₂ : CodingFunction β} {S : Support β} {x : TSet β} (h₁ : χ₁.rel S x) (h₂ : χ₂.rel S x) :
        χ₁.rel χ₂.rel
        theorem ConNF.CodingFunction.ext [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {χ₁ χ₂ : CodingFunction β} (S : Support β) (x : TSet β) (h₁ : χ₁.rel S x) (h₂ : χ₂.rel S x) :
        χ₁ = χ₂
        theorem ConNF.CodingFunction.exists_allPerm_of_rel [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] {χ : CodingFunction β} {S T : Support β} {x y : TSet β} (h₁ : χ.rel S x) (h₂ : χ.rel T y) :
        ∃ (ρ : AllPerm β), ρ S = T ρ x = y
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem ConNF.Tangle.code_eq_code_iff [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] (t₁ t₂ : Tangle β) :
          t₁.code = t₂.code ∃ (ρ : AllPerm β), ρ t₁ = t₂
          @[simp]
          theorem ConNF.Tangle.smul_code [Params] [Level] [CoherentData] {β : TypeIndex} [LeLevel β] (t : Tangle β) (ρ : AllPerm β) :
          (ρ t).code = t.code