Documentation

ConNF.Levels.StrSet

Structural sets #

In this file, we define structural sets, which serve as the environment inside which we will construct the types of our model

Main declarations #

@[irreducible]
Equations
Instances For
    theorem ConNF.StrSet.coe_eq [Params] (α : Λ) :
    StrSet α = ((β : TypeIndex) → β < αSet (StrSet β))
    def ConNF.StrSet.coeEquiv [Params] {α : Λ} :
    StrSet α ((β : TypeIndex) → β < αSet (StrSet β))
    Equations
    Instances For
      theorem ConNF.StrSet.coe_ext_iff' [Params] {α : Λ} {x y : StrSet α} :
      x = y ∀ (β : TypeIndex) ( : β < α) (z : StrSet β), z coeEquiv x β z coeEquiv y β

      Extensionality for structural sets at proper type indices. If two structural sets have the same extensions at every lower type index, then they are the same.

      theorem ConNF.StrSet.strPerm_smul_coe_def [Params] {α : Λ} (π : StrPerm α) (x : StrSet α) :
      strPerm_smul π x = coeEquiv.symm fun (β : TypeIndex) ( : β < α) => strPerm_smul (π ) '' coeEquiv x β
      theorem ConNF.StrSet.strPerm_smul_coe_def' [Params] {α : Λ} (π : StrPerm α) (x : StrSet α) :
      π x = coeEquiv.symm fun (β : TypeIndex) ( : β < α) => strPerm_smul (π ) '' coeEquiv x β
      @[simp]
      theorem ConNF.StrSet.strPerm_smul_coe [Params] {α : Λ} (π : StrPerm α) (x : StrSet α) :
      coeEquiv (π x) = fun (β : TypeIndex) ( : β < α) => π coeEquiv x β
      theorem ConNF.StrSet.mul_strPerm_smul [Params] {α : TypeIndex} (π₁ π₂ : StrPerm α) (x : StrSet α) :
      strPerm_smul (π₁ * π₂) x = strPerm_smul π₁ (strPerm_smul π₂ x)
      theorem ConNF.StrSet.smul_none [Params] {α : Λ} (π : StrPerm α) :
      (π coeEquiv.symm fun (x : TypeIndex) (x_1 : x < α) => ) = coeEquiv.symm fun (x : TypeIndex) (x_1 : x < α) =>

      Notation for typed membership #

      class ConNF.TypedMem [Params] (X : Type u_1) (Y : Type u_2) (β α : outParam TypeIndex) :
      Type (max u_1 u_2)
      • typedMem : β < αXYProp
      Instances
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          def ConNF.typedSubset [Params] (X : Type u_1) {Y : Type u_2} {β α : TypeIndex} [TypedMem X Y β α] (h : β < α) (a b : Y) :
          Equations
          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                instance ConNF.instTypedMemStrSet [Params] {β α : TypeIndex} :
                TypedMem (StrSet β) (StrSet α) β α
                Equations
                • One or more equations did not get rendered due to their size.
                theorem ConNF.StrSet.mem_iff [Params] {α : Λ} {β : TypeIndex} {x : StrSet β} {y : StrSet α} (h : β < α) :
                x ∈[h] y x coeEquiv y β h
                theorem ConNF.StrSet.coe_ext_iff [Params] {α : Λ} {x y : StrSet α} :
                x = y ∀ (β : TypeIndex) ( : β < α) (z : StrSet β), z ∈[] x z ∈[] y

                Extensionality for structural sets at proper type indices. If two structural sets have the same extensions at every lower type index, then they are the same.

                theorem ConNF.StrSet.mem_smul_iff [Params] {α β : TypeIndex} {x : StrSet β} {y : StrSet α} (h : β < α) (π : StrPerm α) :
                x ∈[h] π y (π h)⁻¹ x ∈[h] y