Documentation

ConNF.Counting.CodingFunction

Coding functions #

structure ConNF.CodingFunction [ConNF.Params] (β : ConNF.Λ) [ConNF.ModelData β] :
Instances For
    theorem ConNF.CodingFunction.dom_nonempty [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] (self : ConNF.CodingFunction β) :
    self.decode.Dom.Nonempty
    theorem ConNF.CodingFunction.supports_decode' [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] (self : ConNF.CodingFunction β) (S : ConNF.Support β) (hS : (self.decode S).Dom) :
    MulAction.Supports (ConNF.Allowable β) (ConNF.Enumeration.carrier S) ((self.decode S).get hS)
    theorem ConNF.CodingFunction.dom_iff [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] (self : ConNF.CodingFunction β) (S : ConNF.Support β) (T : ConNF.Support β) (hS : (self.decode S).Dom) :
    (self.decode T).Dom ∃ (ρ : ConNF.Allowable β), T = ρ S
    theorem ConNF.CodingFunction.decode_smul' [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] (self : ConNF.CodingFunction β) (S : ConNF.Support β) (ρ : ConNF.Allowable β) (h₁ : (self.decode S).Dom) (h₂ : (self.decode (ρ S)).Dom) :
    (self.decode (ρ S)).get h₂ = ρ (self.decode S).get h₁
    Equations
    theorem ConNF.CodingFunction.mem_iff [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} {S : ConNF.Support β} :
    S χ (χ.decode S).Dom
    theorem ConNF.CodingFunction.mem_iff_of_mem [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} {S : ConNF.Support β} {T : ConNF.Support β} (h : S χ) :
    T χ ∃ (ρ : ConNF.Allowable β), T = ρ S
    theorem ConNF.CodingFunction.smul_mem [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} {S : ConNF.Support β} (ρ : ConNF.Allowable β) (h : S χ) :
    ρ S χ
    theorem ConNF.CodingFunction.mem_of_smul_mem [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} {S : ConNF.Support β} {ρ : ConNF.Allowable β} (h : ρ S χ) :
    S χ
    theorem ConNF.CodingFunction.exists_mem [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] (χ : ConNF.CodingFunction β) :
    ∃ (S : ConNF.Support β), S χ
    theorem ConNF.CodingFunction.supports_decode [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} (S : ConNF.Support β) (hS : S χ) :
    theorem ConNF.CodingFunction.decode_smul [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} (S : ConNF.Support β) (ρ : ConNF.Allowable β) (h : ρ S χ) :
    (χ.decode (ρ S)).get h = ρ (χ.decode S).get
    theorem ConNF.CodingFunction.ext [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ₁ : ConNF.CodingFunction β} {χ₂ : ConNF.CodingFunction β} (S : ConNF.Support β) (h₁ : S χ₁) (h₂ : S χ₂) (h : (χ₁.decode S).get h₁ = (χ₂.decode S).get h₂) :
    χ₁ = χ₂

    Two coding functions are equal if they decode a single ordered support to the same tangle.

    theorem ConNF.CodingFunction.decode_congr [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} {S₁ : ConNF.Support β} {S₂ : ConNF.Support β} {h₁ : S₁ χ} {h₂ : S₂ χ} (h : S₁ = S₂) :
    (χ.decode S₁).get h₁ = (χ.decode S₂).get h₂

    Produce a coding function for a given ordered support and tangle it supports.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem ConNF.CodingFunction.mem_code [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {S : ConNF.Support β} {t : ConNF.TSet β} {h : MulAction.Supports (ConNF.Allowable β) (ConNF.Enumeration.carrier S) t} (T : ConNF.Support β) :
      T ConNF.CodingFunction.code S t h ∃ (ρ : ConNF.Allowable β), T = ρ S
      theorem ConNF.CodingFunction.eq_code [ConNF.Params] {β : ConNF.Λ} [ConNF.ModelData β] {χ : ConNF.CodingFunction β} {S : ConNF.Support β} (h : S χ) :
      χ = ConNF.CodingFunction.code S ((χ.decode S).get h)

      Every coding function can be obtained by invoking code with an ordered support in its domain.