Documentation

ConNF.Model.Basic

def ConNF.mem [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (h : β < α) (tβ : ConNF.TSet β) (tα : ConNF.TSet α) :
Equations
  • ( ∈[h] ) = (ConNF.toStructSet ConNF.StructSet.ofCoe (ConNF.toStructSet ) β )
Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem ConNF.tSet_mk_aux [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : Set (ConNF.TSet β)) (hs : ∃ (S : Set (ConNF.Address α)), ConNF.Small S ∀ (ρ : ConNF.Allowable α), (cS, ρ c = c)(ConNF.cons ) ρ s = s) :
      ∃ (S : Set (ConNF.Address α)), ConNF.Small S ∀ (ρ : ConNF.NewAllowable), (cS, ρ c = c)ρ β s = s
      def ConNF.Symmetric [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : Set (ConNF.TSet β)) :
      Equations
      Instances For
        theorem ConNF.Symmetric.ofSubset [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : Set (ConNF.TSet β)) :
        (∃ (S : Set (ConNF.Address α)), ConNF.Small S ∀ (ρ : ConNF.Allowable α), (cS, ρ c = c)(ConNF.cons ) ρ s s)ConNF.Symmetric s
        def ConNF.ModelData.TSet.mk [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : Set (ConNF.TSet β)) (hs : ConNF.Symmetric s) :
        Equations
        Instances For
          theorem ConNF.ModelData.TSet.toStructSet_eq [ConNF.Params] {α : ConNF.Λ} (t : ConNF.TSet α) :
          ConNF.toStructSet t = ConNF.NewTSet.toStructSet ((ConNF.tSetEquiv α) t)
          theorem ConNF.ModelData.TSet.mem_tSetEquiv_iff [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : ConNF.TSet β) (t : ConNF.TSet α) :
          s ∈[] t ConNF.toStructSet s ConNF.StructSet.ofCoe (ConNF.NewTSet.toStructSet ((ConNF.tSetEquiv α) t)) β
          theorem ConNF.ModelData.TSet.ofCoe_toStructSet_apply_eq [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (t : ConNF.TSet α) :
          ConNF.StructSet.ofCoe (ConNF.toStructSet t) β = {p : ConNF.StructSet β | s(((ConNF.tSetEquiv α) t)).members β, ConNF.toStructSet s = p}
          @[simp]
          theorem ConNF.ModelData.TSet.mem_mk_iff [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : Set (ConNF.TSet β)) (hs : ConNF.Symmetric s) (t : ConNF.TSet β) :
          theorem ConNF.ModelData.TSet.eq_toStructSet_of_mem [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (t₁ : ConNF.TSet α) (t₂ : ConNF.StructSet β) :
          t₂ ConNF.StructSet.ofCoe (ConNF.NewTSet.toStructSet ((ConNF.tSetEquiv α) t₁)) β ∃ (t₂' : ConNF.TSet β), t₂ = ConNF.toStructSet t₂'
          theorem ConNF.ModelData.TSet.ext [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (t₁ : ConNF.TSet α) (t₂ : ConNF.TSet α) :
          (∀ (s : ConNF.TSet β), s ∈[] t₁ s ∈[] t₂)t₁ = t₂
          theorem ConNF.ModelData.TSet.smul_mem_smul [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : ConNF.TSet β) (t : ConNF.TSet α) (ρ : ConNF.Allowable α) (h : s ∈[] t) :
          (ConNF.cons ) ρ s ∈[] ρ t
          theorem ConNF.ModelData.TSet.smul_mem_smul_iff [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : ConNF.TSet β) (t : ConNF.TSet α) (ρ : ConNF.Allowable α) :
          (ConNF.cons ) ρ s ∈[] ρ t s ∈[] t
          theorem ConNF.ModelData.TSet.smul_mem_iff [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : ConNF.TSet β) (t : ConNF.TSet α) (ρ : ConNF.Allowable α) :
          (ConNF.cons ) ρ s ∈[] t s ∈[] ρ⁻¹ t
          theorem ConNF.ModelData.TSet.mem_smul_iff [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (s : ConNF.TSet β) (t : ConNF.TSet α) (ρ : ConNF.Allowable α) :
          s ∈[] ρ t ((ConNF.cons ) ρ)⁻¹ s ∈[] t
          theorem ConNF.ModelData.TSet.induction [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} (hβ : β < α) (t : ConNF.TSet α) :
          ∃ (s : Set (ConNF.TSet β)) (hs : ConNF.Symmetric s), t = ConNF.ModelData.TSet.mk s hs
          theorem ConNF.Small.symmetric [ConNF.Params] {β : ConNF.Λ} {α : ConNF.Λ} {s : Set (ConNF.TSet β)} (hs : ConNF.Small s) (hβ : β < α) :