Documentation

ConNF.Strong.CodingFunction

Coding functions #

In this file, we define coding functions.

Main declarations #

Equations
Instances For
    Instances For
      theorem ConNF.CodingFunction.ext' [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] {χ₁ χ₂ : ConNF.CodingFunction β} (h : ∀ (S : ConNF.Support β) (x : ConNF.TSet β), χ₁.rel S x χ₂.rel S x) :
      χ₁ = χ₂
      theorem ConNF.CodingFunction.ext_aux [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] {χ₁ χ₂ : ConNF.CodingFunction β} {S : ConNF.Support β} {x : ConNF.TSet β} (h₁ : χ₁.rel S x) (h₂ : χ₂.rel S x) :
      χ₁.rel χ₂.rel
      theorem ConNF.CodingFunction.ext [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] {χ₁ χ₂ : ConNF.CodingFunction β} (S : ConNF.Support β) (x : ConNF.TSet β) (h₁ : χ₁.rel S x) (h₂ : χ₂.rel S x) :
      χ₁ = χ₂
      theorem ConNF.CodingFunction.exists_allPerm_of_rel [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] {χ : ConNF.CodingFunction β} {S T : ConNF.Support β} {x y : ConNF.TSet β} (h₁ : χ.rel S x) (h₂ : χ.rel T y) :
      ∃ (ρ : ConNF.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 [ConNF.Params] [ConNF.Level] [ConNF.CoherentData] {β : ConNF.TypeIndex} [ConNF.LeLevel β] (t₁ t₂ : ConNF.Tangle β) :
        t₁.code = t₂.code ∃ (ρ : ConNF.AllPerm β), ρ t₁ = t₂