Construction of model data #
In this file, we construct model data at type α
, given that it is defined at all types below α
.
Main declarations #
ConNF.foo
: Something new.
Equations
- ConNF.instMulNewPerm = { mul := fun (ρ₁ ρ₂ : ConNF.NewPerm) => { sderiv := fun (β : ConNF.TypeIndex) (x : ConNF.LtLevel β) => ρ₁.sderiv β * ρ₂.sderiv β, smul_fuzz' := ⋯ } }
Equations
- ConNF.instOneNewPerm = { one := { sderiv := fun (x : ConNF.TypeIndex) (x_1 : ConNF.LtLevel x) => 1, smul_fuzz' := ⋯ } }
Equations
- ConNF.instInvNewPerm = { inv := fun (ρ : ConNF.NewPerm) => { sderiv := fun (β : ConNF.TypeIndex) (x : ConNF.LtLevel β) => (ρ.sderiv β)⁻¹, smul_fuzz' := ⋯ } }
Equations
Equations
- ConNF.instSMulNewPermCode = { smul := fun (ρ : ConNF.NewPerm) (c : ConNF.Code) => ConNF.Code.mk c.β (ρ.sderiv c.β • c.s) ⋯ }
Equations
theorem
ConNF.Represents.smul
[Params]
[Level]
[LtData]
{c d : Code}
(h : Represents c d)
(ρ : NewPerm)
:
Represents (ρ • c) (ρ • d)
theorem
ConNF.NewPerm.forget_def
[Params]
[Level]
[LtData]
(ρ : NewPerm)
(A : ↑α ↝ ⊥)
:
ρᵁ A = Path.recScoderiv (motive := fun (β : TypeIndex) (x : β ↝ ⊥) => β ≠ ⊥ → β ≤ ↑α → BasePerm) (fun (h : ⊥ ≠ ⊥) => ⋯.elim)
(fun (_β γ : TypeIndex) (B : γ ↝ ⊥) (hγβ : γ < _β)
(x : (fun (β : TypeIndex) (x : β ↝ ⊥) => β ≠ ⊥ → β ≤ ↑α → BasePerm) γ B) (x : _β ≠ ⊥) (hβα : _β ≤ ↑α) =>
(ρ.sderiv γ)ᵁ B)
A ⋯ ⋯
Equations
- ConNF.instSMulNewPermNewSet = { smul := fun (ρ : ConNF.NewPerm) (x : ConNF.NewSet) => { c := ρ • x.c, hc := ⋯, hS := ⋯ } }
Equations
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
Equations
- ConNF.newModelData = ConNF.ModelData.mk ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Instances For
Equations
- N.code = ConNF.Code.mk ⊥ {x : ConNF.TSet ⊥ | ConNF.StrSet.botEquiv xᵁ ∈ Nᴬ} ⋯
Instances For
Equations
- ConNF.newTyped N = N.code.toSet ⋯
Instances For
Equations
- ConNF.newSingletonCode x = ConNF.Code.mk ↑γ {x} ⋯
Instances For
Equations
Instances For
Equations
Instances For
Equations
- ConNF.newPosition h = { pos := { toFun := ConNF.funOfDeny h ConNF.newPositionDeny ⋯, inj' := ⋯ } }
Instances For
def
ConNF.newTypedNearLitters
[Params]
[Level]
[LtData]
(h : Cardinal.mk (Tangle ↑α) ≤ Cardinal.mk μ)
:
Equations
- ConNF.newTypedNearLitters h = { typed := some ∘ ConNF.newTyped, typed_injective := ⋯, pos_le_pos_of_typed := ⋯, smul_typed := ⋯ }