Documentation

ConNF.Counting.BaseCoding

Coding the base type #

In this file, we prove a consequence of freedom of action for : a base support can support at most 2 ^ #κ-many different sets of atoms under the action of base permutations.

Main declarations #

Equations
Instances For
    theorem ConNF.addAtom'_atoms_rel [Params] (S : BaseSupport) (a : Atom) (i : κ) (b : Atom) :
    (addAtom' S a).rel i b S.rel i b b = a i = S.bound
    Equations
    Instances For
      @[simp]
      theorem ConNF.addAtom_convAtoms [Params] (S : BaseSupport) (a₁ a₂ : Atom) (A : ) :
      convAtoms (addAtom S a₁) (addAtom S a₂) A = fun (a₃ a₄ : Atom) => a₃ = a₄ a₃ S a₃ = a₁ a₄ = a₂
      @[simp]
      theorem ConNF.addAtom_convNearLitters [Params] (S : BaseSupport) (a₁ a₂ : Atom) (A : ) :
      convNearLitters (addAtom S a₁) (addAtom S a₂) A = fun (N₁ N₂ : NearLitter) => N₁ = N₂ N₁ S
      theorem ConNF.addAtom_sameSpecLe [Params] [Level] [CoherentData] {S : BaseSupport} {a₁ a₂ : Atom} (ha₁ : a₁S) (ha₂ : a₂S) (ha : NS, a₁ N a₂ N) :
      SameSpecLE (addAtom S a₁) (addAtom S a₂)
      theorem ConNF.addAtom_spec_eq_spec [Params] [Level] [CoherentData] {S : BaseSupport} {a₁ a₂ : Atom} (ha₁ : a₁S) (ha₂ : a₂S) (ha : NS, a₁ N a₂ N) :
      (addAtom S a₁).spec = (addAtom S a₂).spec
      theorem ConNF.exists_swap [Params] [Level] [CoherentData] {S : BaseSupport} (h : S.Closed) {a₁ a₂ : Atom} (ha₁ : a₁S) (ha₂ : a₂S) (ha : NS, a₁ N a₂ N) :
      ∃ (π : BasePerm), π S = S π a₁ = a₂
      theorem ConNF.mem_iff_mem_of_supports [Params] [Level] [CoherentData] {S : BaseSupport} (h : S.Closed) {s : Set Atom} (hs : ∀ (π : BasePerm), π S = Sπ s = s) {a₁ a₂ : Atom} (h₁ : a₁S) (h₂ : a₂S) (ha : NS, a₁ N a₂ N) :
      a₁ s a₂ s
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem ConNF.subset_of_information_eq [Params] [Level] [CoherentData] {S : BaseSupport} (hS : S.Closed) {s t : Set Atom} (hs : ∀ (π : BasePerm), π S = Sπ s = s) (ht : ∀ (π : BasePerm), π S = Sπ t = t) (h : information S s = information S t) :
          s t
          theorem ConNF.eq_of_information_eq [Params] [Level] [CoherentData] {S : BaseSupport} (hS : S.Closed) {s t : Set Atom} (hs : ∀ (π : BasePerm), π S = Sπ s = s) (ht : ∀ (π : BasePerm), π S = Sπ t = t) (h : information S s = information S t) :
          s = t
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For