Documentation

ConNF.FOA.Inflexible

New file #

In this file...

Main declarations #

Instances For
    theorem ConNF.InflexiblePath.ext {inst✝ : ConNF.Params} {β : ConNF.TypeIndex} {x y : ConNF.InflexiblePath β} (γ : x = y) (δ : x = y) (ε : x = y) (A : HEq x.A y.A) :
    x = y
    Equations
    • One or more equations did not get rendered due to their size.
    @[simp]
    theorem ConNF.InflexiblePath.coderiv_A [ConNF.Params] {β β' : ConNF.TypeIndex} (P : ConNF.InflexiblePath β) (B : β' β) :
    (P B).A = B P.A
    Equations
    Instances For
      theorem ConNF.inflexiblePath_subsingleton [ConNF.Params] {β : ConNF.TypeIndex} [ConNF.Level] [ConNF.CoherentData] [ConNF.LeLevel β] {A : β } {L : ConNF.Litter} {P₁ P₂ : ConNF.InflexiblePath β} {t₁ : ConNF.Tangle P₁} {t₂ : ConNF.Tangle P₂} (hP₁ : A = P₁.A ↘.) (hP₂ : A = P₂.A ↘.) (ht₁ : L = ConNF.fuzz t₁) (ht₂ : L = ConNF.fuzz t₂) :
      P₁ = P₂
      Equations
      Instances For