instance
ConNF.instCoderivativeInflexiblePath
[Params]
{β β' : TypeIndex}
:
Coderivative (InflexiblePath β) (InflexiblePath β') β' β
Equations
- One or more equations did not get rendered due to their size.
instance
ConNF.instLeLevelSomeΛγ
[Params]
{β : TypeIndex}
[Level]
[LeLevel β]
(P : InflexiblePath β)
:
instance
ConNF.instLtLevelδOfLeLevel
[Params]
{β : TypeIndex}
[Level]
[LeLevel β]
(P : InflexiblePath β)
:
instance
ConNF.instLtLevelSomeΛεOfLeLevel
[Params]
{β : TypeIndex}
[Level]
[LeLevel β]
(P : InflexiblePath β)
:
def
ConNF.Inflexible
[Params]
{β : TypeIndex}
[Level]
[CoherentData]
[LeLevel β]
(A : β ↝ ⊥)
(L : Litter)
:
Equations
- ConNF.Inflexible A L = ∃ (P : ConNF.InflexiblePath β) (t : ConNF.Tangle P.δ), A = P.A ↘ ⋯ ↘. ∧ L = ConNF.fuzz ⋯ t
Instances For
theorem
ConNF.inflexible_deriv
[Params]
{β : TypeIndex}
[Level]
[CoherentData]
[LeLevel β]
{A : β ↝ ⊥}
{L : Litter}
(h : Inflexible A L)
{β' : TypeIndex}
[LeLevel β']
(B : β' ↝ β)
:
Inflexible (B ⇘ A) L