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 #
ConNF.StrSet
: The type family of structural sets.
@[irreducible]
Equations
- ConNF.StrSet none = ConNF.Atom
- ConNF.StrSet (some α) = ((β : ConNF.TypeIndex) → β < ↑α → Set (ConNF.StrSet β))
Instances For
Equations
Instances For
Equations
Instances For
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.
@[irreducible]
Equations
- ConNF.StrSet.strPerm_smul π x_3 = ConNF.StrSet.botEquiv.symm (π ConNF.Path.nil • ConNF.StrSet.botEquiv x_3)
- ConNF.StrSet.strPerm_smul π x_3 = ConNF.StrSet.coeEquiv.symm fun (β : ConNF.TypeIndex) (hβ : β < ↑α) => ConNF.StrSet.strPerm_smul (π ↘ hβ) '' ConNF.StrSet.coeEquiv x_3 β hβ
Instances For
Equations
- ConNF.StrSet.instSMulStrPerm = { smul := ConNF.StrSet.strPerm_smul }
Equations
Notation for typed membership #
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ConNF.«term_∈'_» = Lean.ParserDescr.trailingNode `ConNF.«term_∈'_» 50 50 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ∈' ") (Lean.ParserDescr.cat `term 50))
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
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.