Documentation

ConNF.Counting.Recode

Raising supports to higher levels #

def ConNF.raiseIndex [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} (hγ : γ < β) (A : ConNF.ExtendedIndex γ) :
Equations
Instances For
    def ConNF.raise [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} (hγ : γ < β) (c : ConNF.Address γ) :
    Equations
    Instances For
      @[simp]
      theorem ConNF.raise_path [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} (hγ : γ < β) (c : ConNF.Address γ) :
      (ConNF.raise c).path = ConNF.raiseIndex c.path
      @[simp]
      theorem ConNF.raise_value [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} (hγ : γ < β) (c : ConNF.Address γ) :
      (ConNF.raise c).value = c.value
      theorem ConNF.raiseIndex_injective [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} (hγ : γ < β) {A : ConNF.ExtendedIndex γ} {B : ConNF.ExtendedIndex γ} (h : ConNF.raiseIndex A = ConNF.raiseIndex B) :
      A = B
      theorem Quiver.Path.comp_injective' {V : Type u_1} [Quiver V] {a : V} {b : V} {c : V} {d : V} {p₁ : Quiver.Path a b} {p₂ : Quiver.Path a c} {q₁ : Quiver.Path b d} {q₂ : Quiver.Path c d} (h₁ : p₁.length = p₂.length) (h₂ : p₁.comp q₁ = p₂.comp q₂) :
      b = c
      theorem ConNF.raiseIndex_index_injective [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} {δ : ConNF.Λ} (hγ : γ < β) (hδ : δ < β) {A : ConNF.ExtendedIndex γ} {B : ConNF.ExtendedIndex δ} (h : ConNF.raiseIndex A = ConNF.raiseIndex B) :
      γ = δ
      theorem ConNF.raise_injective [ConNF.Params] {β : ConNF.Λ} {γ : ConNF.Λ} (hγ : γ < β) {c : ConNF.Address γ} {d : ConNF.Address γ} (h : ConNF.raise c = ConNF.raise d) :
      c = d
      theorem ConNF.smul_raise_eq_iff [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (c : ConNF.Address γ) (ρ : ConNF.Allowable β) :
      def ConNF.Appears [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] (hγ : γ < β) (s : Set (ConNF.StructSet γ)) :

      A set s of γ-structSets appears at level α if it occurs as the γ-extension of some α-tangle.

      Equations
      Instances For
        def ConNF.AppearsRaised [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] (hγ : γ < β) (χs : Set (ConNF.CodingFunction β)) (U : ConNF.Support β) :
        Equations
        Instances For
          noncomputable def ConNF.decodeRaised [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] (hγ : γ < β) (χs : Set (ConNF.CodingFunction β)) (U : ConNF.Support β) (hU : ConNF.AppearsRaised χs U) :
          Equations
          Instances For

            We now aim to show that decodeRaised is a coding function.

            theorem ConNF.decodeRaised_spec [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] (hγ : γ < β) (χs : Set (ConNF.CodingFunction β)) (U : ConNF.Support β) (hU : ConNF.AppearsRaised χs U) :
            ConNF.StructSet.ofCoe (ConNF.toStructSet (ConNF.decodeRaised χs U hU)) (γ) = {u : ConNF.StructSet γ | χχs, VU, ∃ (hV : V χ), u ConNF.StructSet.ofCoe (ConNF.toStructSet ((χ.decode V).get hV)) (γ) }
            theorem ConNF.appearsRaised_smul [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] (hγ : γ < β) {χs : Set (ConNF.CodingFunction β)} (U : ConNF.Support β) (hU : ConNF.AppearsRaised χs U) (ρ : ConNF.Allowable β) :
            ConNF.AppearsRaised χs (ρ U)
            theorem ConNF.decodeRaised_smul [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) {χs : Set (ConNF.CodingFunction β)} (U : ConNF.Support β) (hU : ConNF.AppearsRaised χs U) (ρ : ConNF.Allowable β) :
            ConNF.decodeRaised χs (ρ U) = ρ ConNF.decodeRaised χs U hU
            def ConNF.tangleExtension [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (t : ConNF.TSet β) :
            Set (ConNF.TSet γ)

            The tangles in the γ-extension of a given β-tangle.

            Equations
            Instances For
              noncomputable def ConNF.raisedSupport [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (u : ConNF.TSet γ) :

              A support for a γ-tangle, expressed as a set of β-support conditions.

              Equations
              Instances For
                theorem ConNF.le_raisedSupport [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (u : ConNF.TSet γ) :
                theorem ConNF.raisedSupport_supports [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (u : ConNF.TSet γ) :
                noncomputable def ConNF.raiseSingleton [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (u : ConNF.TSet γ) :
                Equations
                Instances For
                  def ConNF.RaisedSingleton [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) :
                  Equations
                  Instances For
                    theorem ConNF.smul_raise_eq [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (ρ : ConNF.Allowable β) (c : ConNF.Address γ) :
                    theorem ConNF.smul_image_raise_eq [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (ρ : ConNF.Allowable β) (T : ConNF.Support γ) :
                    def ConNF.raiseSingletons [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) :

                    Take the γ-extension of t, treated as a set of α-level singletons, and turn them into coding functions.

                    Equations
                    Instances For
                      theorem ConNF.raiseSingletons_subset_range [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) {S : ConNF.Support β} {t : ConNF.TSet β} :
                      ConNF.raiseSingletons S t Set.range Subtype.val
                      theorem ConNF.smul_reducedSupport_eq [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (v : ConNF.TSet γ) (ρ : ConNF.Allowable β) (hUV : S ρ ConNF.raisedSupport S v) (c : ConNF.Address β) (hc : c S) :
                      ρ c = c
                      theorem ConNF.raiseSingletons_reducedSupport [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) :
                      {u : ConNF.StructSet γ | χConNF.raiseSingletons S t, VS, ∃ (hV : V χ), u ConNF.StructSet.ofCoe (ConNF.toStructSet ((χ.decode V).get hV)) (γ) } = ConNF.StructSet.ofCoe (ConNF.toStructSet t) (γ)
                      theorem ConNF.appearsRaised_raiseSingletons [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) :
                      theorem ConNF.decodeRaised_raiseSingletons [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) :
                      noncomputable def ConNF.raisedCodingFunction [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (χs : Set (ConNF.CodingFunction β)) (o : ConNF.SupportOrbit β) (ho : Uo, ConNF.AppearsRaised χs U) (ho' : ∀ (U : ConNF.Support β) (hU : U o), MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c U} (ConNF.decodeRaised χs U )) :
                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        theorem ConNF.decode_raisedCodingFunction [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (χs : Set (ConNF.CodingFunction β)) (o : ConNF.SupportOrbit β) (ho : Uo, ConNF.AppearsRaised χs U) (ho' : ∀ (U : ConNF.Support β) (hU : U o), MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c U} (ConNF.decodeRaised χs U )) (U : ConNF.Support β) (hU : U ConNF.raisedCodingFunction χs o ho ho') :
                        ((ConNF.raisedCodingFunction χs o ho ho').decode U).get hU = ConNF.decodeRaised χs U
                        theorem ConNF.mem_raisedCodingFunction_iff [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (χs : Set (ConNF.CodingFunction β)) (o : ConNF.SupportOrbit β) (ho : Uo, ConNF.AppearsRaised χs U) (ho' : ∀ (U : ConNF.Support β) (hU : U o), MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c U} (ConNF.decodeRaised χs U )) (U : ConNF.Support β) :
                        U ConNF.raisedCodingFunction χs o ho ho' U o
                        theorem ConNF.appearsRaised_of_mem_orbit [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) (U : ConNF.Support β) (hU : U ConNF.SupportOrbit.mk S) :
                        theorem ConNF.supports_decodeRaised_of_mem_orbit [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) (U : ConNF.Support β) (hU : U ConNF.SupportOrbit.mk S) :
                        noncomputable def ConNF.recode [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) :

                        Converts a tangle to a coding class by going via raisedCodingFunction γ.

                        Equations
                        Instances For
                          theorem ConNF.decode_recode [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) :
                          ((ConNF.recode S t hSt).decode S).get = t
                          theorem ConNF.recode_eq [ConNF.Params] [ConNF.Level] [ConNF.BasePositions] [ConNF.CountingAssumptions] {β : ConNF.Λ} {γ : ConNF.Λ} [ConNF.LeLevel β] [ConNF.LeLevel γ] (hγ : γ < β) (S : ConNF.Support β) (t : ConNF.TSet β) (hSt : MulAction.Supports (ConNF.Allowable β) {c : ConNF.Address β | c S} t) :

                          The recode function yields the original coding function on t.