Documentation

ConNF.FOA.Inflexible

New file #

In this file...

Main declarations #

Instances For
    theorem ConNF.InflexiblePath.ext {inst✝ : Params} {β : TypeIndex} {x y : 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 [Params] {β β' : TypeIndex} (P : InflexiblePath β) (B : β' β) :
    (P B).A = B P.A
    Equations
    Instances For
      theorem ConNF.inflexible_iff [Params] {β : TypeIndex} [Level] [CoherentData] [LeLevel β] (A : β ) (L : Litter) :
      Inflexible A L ∃ (P : InflexiblePath β) (t : Tangle P.δ), A = P.A ↘. L = fuzz t
      theorem ConNF.not_inflexible_iff [Params] {β : TypeIndex} [Level] [CoherentData] [LeLevel β] (A : β ) (L : Litter) :
      ¬Inflexible A L ∀ (P : InflexiblePath β) (t : Tangle P.δ), A = P.A ↘.L fuzz t
      theorem ConNF.inflexible_deriv [Params] {β : TypeIndex} [Level] [CoherentData] [LeLevel β] {A : β } {L : Litter} (h : Inflexible A L) {β' : TypeIndex} [LeLevel β'] (B : β' β) :
      Inflexible (B A) L
      theorem ConNF.inflexible_cases [Params] {β : TypeIndex} [Level] [CoherentData] [LeLevel β] (A : β ) (L : Litter) :
      (∃ (P : InflexiblePath β) (t : Tangle P.δ), A = P.A ↘. L = fuzz t) ¬Inflexible A L
      theorem ConNF.inflexiblePath_subsingleton [Params] {β : TypeIndex} [Level] [CoherentData] [LeLevel β] {A : β } {L : Litter} {P₁ P₂ : InflexiblePath β} {t₁ : Tangle P₁.δ} {t₂ : Tangle P₂.δ} (hP₁ : A = P₁.A ↘.) (hP₂ : A = P₂.A ↘.) (ht₁ : L = fuzz t₁) (ht₂ : L = fuzz t₂) :
      P₁ = P₂
      Equations
      Instances For