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 #
ConNF.foo
: Something new.
Equations
- ConNF.addAtom' S a = { atoms := Sᴬ + ConNF.Enumeration.singleton a, nearLitters := Sᴺ }
Instances For
Equations
Instances For
@[simp]
Equations
- ConNF.addAtom S a = ConNF.Support.ofBase (ConNF.addAtom' S a)
Instances For
theorem
ConNF.addAtom_strong
[Params]
[Level]
[CoherentData]
(S : BaseSupport)
(a : Atom)
(hS : S.Closed)
:
@[simp]
theorem
ConNF.addAtom_sameSpecLe
[Params]
[Level]
[CoherentData]
{S : BaseSupport}
{a₁ a₂ : Atom}
(ha₁ : a₁ ∉ Sᴬ)
(ha₂ : a₂ ∉ Sᴬ)
(ha : ∀ N ∈ Sᴺ, a₁ ∈ Nᴬ ↔ a₂ ∈ Nᴬ)
:
SameSpecLE (addAtom S a₁) (addAtom S a₂)
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)
:
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)
:
theorem
ConNF.card_supports_le_of_closed'
[Params]
[Level]
[CoherentData]
{S : BaseSupport}
(hS : S.Closed)
:
theorem
ConNF.card_supports_le_of_closed
[Params]
[Level]
[CoherentData]
{S : BaseSupport}
(hS : S.Closed)
: