Documentation

ConNF.ModelData.ModelData

Model data #

In this file, we define what model data at a type index means.

Main declarations #

class ConNF.PreModelData [Params] (α : TypeIndex) :
Type (u + 1)

The same as ModelData but without the propositions.

Instances
    structure ConNF.Support.Supports [Params] {X : Type u_1} {α : TypeIndex} [PreModelData α] [MulAction (AllPerm α) X] (S : Support α) (x : X) :
    Instances For
      theorem ConNF.Support.Supports.mono [Params] {X : Type u_1} {α : TypeIndex} [PreModelData α] [MulAction (AllPerm α) X] {S T : Support α} {x : X} (hS : S.Supports x) (h : S T) (hT : α = T = Enumeration.empty) :
      class ConNF.ModelData [Params] (α : TypeIndex) extends ConNF.PreModelData α :
      Type (u + 1)
      Instances
        theorem ConNF.tSetForget_injective [Params] {α : TypeIndex} [ModelData α] {x₁ x₂ : TSet α} (h : x₁ = x₂) :
        x₁ = x₂
        theorem ConNF.allPermForget_injective [Params] {α : TypeIndex} [ModelData α] {ρ₁ ρ₂ : AllPerm α} (h : ρ₁ = ρ₂) :
        ρ₁ = ρ₂
        @[simp]
        @[simp]
        theorem ConNF.allPermForget_npow [Params] {α : TypeIndex} [ModelData α] (ρ : AllPerm α) (n : ) :
        (ρ ^ n) = ρ ^ n
        @[simp]
        theorem ConNF.allPermForget_zpow [Params] {α : TypeIndex} [ModelData α] (ρ : AllPerm α) (n : ) :
        (ρ ^ n) = ρ ^ n
        theorem ConNF.Support.Supports.smul_eq_smul [Params] {X : Type u_1} {α : TypeIndex} [ModelData α] [MulAction (AllPerm α) X] {S : Support α} {x : X} (h : S.Supports x) {ρ₁ ρ₂ : AllPerm α} ( : ρ₁ S = ρ₂ S) :
        ρ₁ x = ρ₂ x
        theorem ConNF.Support.Supports.smul_eq_of_smul_eq [Params] {X : Type u_1} {α : TypeIndex} [ModelData α] [MulAction (AllPerm α) X] {S : Support α} {x : X} (h : S.Supports x) {ρ : AllPerm α} ( : ρ S = S) :
        ρ x = x
        theorem ConNF.Support.Supports.smul [Params] {X : Type u_1} {α : TypeIndex} [ModelData α] [MulAction (AllPerm α) X] {S : Support α} {x : X} (h : S.Supports x) (ρ : AllPerm α) :
        (ρ S).Supports (ρ x)
        instance ConNF.instTypedMemTSet [Params] {β α : TypeIndex} [ModelData β] [ModelData α] :
        TypedMem (TSet β) (TSet α) β α
        Equations
        theorem ConNF.TSet.forget_mem_forget [Params] {β α : TypeIndex} [ModelData β] [ModelData α] (h : β < α) {x : TSet β} {y : TSet α} :
        structure ConNF.Tangle [Params] (α : TypeIndex) [ModelData α] :
        Instances For
          theorem ConNF.Tangle.ext {inst✝ : Params} {α : TypeIndex} {inst✝¹ : ModelData α} {x y : Tangle α} (set : x.set = y.set) (support : x.support = y.support) :
          x = y
          Equations
          @[simp]
          theorem ConNF.Tangle.smul_set [Params] {α : TypeIndex} [ModelData α] (ρ : AllPerm α) (t : Tangle α) :
          (ρ t).set = ρ t.set
          @[simp]
          theorem ConNF.Tangle.smul_support [Params] {α : TypeIndex} [ModelData α] (ρ : AllPerm α) (t : Tangle α) :
          (ρ t).support = ρ t.support
          theorem ConNF.Tangle.smul_eq_smul [Params] {α : TypeIndex} [ModelData α] {ρ₁ ρ₂ : AllPerm α} {t : Tangle α} (h : ρ₁ t.support = ρ₂ t.support) :
          ρ₁ t = ρ₂ t
          theorem ConNF.Tangle.smul_eq [Params] {α : TypeIndex} [ModelData α] {ρ : AllPerm α} {t : Tangle α} (h : ρ t.support = t.support) :
          ρ t = t
          theorem ConNF.Tangle.smul_atom_eq_of_mem_support [Params] {α : TypeIndex} [ModelData α] {ρ₁ ρ₂ : AllPerm α} {t : Tangle α} (h : ρ₁ t = ρ₂ t) {a : Atom} {A : α } (ha : a (t.support ⇘. A)) :
          ρ₁ A a = ρ₂ A a
          theorem ConNF.Tangle.smul_nearLitter_eq_of_mem_support [Params] {α : TypeIndex} [ModelData α] {ρ₁ ρ₂ : AllPerm α} {t : Tangle α} (h : ρ₁ t = ρ₂ t) {N : NearLitter} {A : α } (hN : N (t.support ⇘. A)) :
          ρ₁ A N = ρ₂ A N

          Criteria for supports #

          theorem ConNF.Support.supports_coe [Params] {α : Λ} {X : Type u_1} [PreModelData α] [MulAction (AllPerm α) X] (S : Support α) (x : X) (h : ∀ (ρ : AllPerm α), (∀ (A : α ), a ∈ (S ⇘. A), ρ A a = a)(∀ (A : α ), N ∈ (S ⇘. A), ρ A N = N)ρ x = x) :
          theorem ConNF.Support.supports_bot [Params] {X : Type u_1} [PreModelData ] [MulAction (AllPerm ) X] (E : Enumeration ( × Atom)) (x : X) (h : ∀ (ρ : AllPerm ), (∀ (A : ) (x : Atom), (A, x) Eρ A x = x)ρ x = x) :
          { atoms := E, nearLitters := Enumeration.empty }.Supports x

          Model data at level #

          Equations
          Instances For