def
ConNF.constructSingleton
[Params]
{α : Λ}
(M : (β : Λ) → ↑β < ↑α → Motive β)
(H : (β : Λ) → (h : ↑β < ↑α) → Hypothesis (M β h) fun (γ : Λ) (h' : ↑γ < ↑β) => M γ ⋯)
{β : Λ}
(h : ↑β < ↑α)
(x : TSet ↑β)
:
TSet ↑α
Equations
- ConNF.constructSingleton M H h x = some (ConNF.newSingleton x)
Instances For
theorem
ConNF.constructMotive_allPerm_of_smul_fuzz
[Params]
{α : Λ}
(M : (β : Λ) → ↑β < ↑α → Motive β)
(H : (β : Λ) → (h : ↑β < ↑α) → Hypothesis (M β h) fun (γ : Λ) (h' : ↑γ < ↑β) => M γ ⋯)
(ρs : {β : Λ} → (hβ : ↑β < ↑α) → AllPerm ↑β)
(π : AllPerm ⊥)
:
(∀ {β γ : Λ} (hβ : ↑β < ↑α) (hγ : ↑γ < ↑α) (hδε : ↑β ≠ ↑γ) (t : Tangle ↑β),
(ρs hγ)ᵁ ↘. • fuzz hδε t = fuzz hδε (ρs hβ • t)) →
(∀ {γ : Λ} (hγ : ↑γ < ↑α) (t : Tangle ⊥), (ρs hγ)ᵁ ↘. • fuzz ⋯ t = fuzz ⋯ (π • t)) →
∃ (ρ : AllPerm ↑α),
(∀ (β : Λ) (hβ : ↑β < ↑α), constructAllPermSderiv M H hβ ρ = ρs hβ) ∧ constructAllPermBotSderiv M H ρ = π
def
ConNF.constructHypothesis
[Params]
(α : Λ)
(M : (β : Λ) → ↑β < ↑α → Motive β)
(H : (β : Λ) → (h : ↑β < ↑α) → Hypothesis (M β h) fun (γ : Λ) (h' : ↑γ < ↑β) => M γ ⋯)
:
Hypothesis (constructMotive α M H) M
Equations
- One or more equations did not get rendered due to their size.