Documentation

ConNF.Model.InductionStatement

New file #

In this file...

Main declarations #

structure ConNF.Motive [ConNF.Params] (α : ConNF.Λ) :
Type (u + 1)
Instances For
    Equations
    Instances For
      theorem ConNF.pos_tangle_bot [ConNF.Params] {D : ConNF.ModelData } (t : ConNF.Tangle ) (a : ConNF.Atom) (A : ) (ha : a (t.support ⇘. A)) :
      ConNF.pos a < ConNF.pos t
      structure ConNF.Hypothesis [ConNF.Params] {α : ConNF.Λ} (M : ConNF.Motive α) (N : (β : ConNF.Λ) → β < αConNF.Motive β) :
      Instances For
        def ConNF.castTSet [ConNF.Params] {α β : ConNF.TypeIndex} {D₁ : ConNF.ModelData α} {D₂ : ConNF.ModelData β} (h₁ : α = β) (h₂ : HEq D₁ D₂) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          def ConNF.castAllPerm [ConNF.Params] {α β : ConNF.TypeIndex} {D₁ : ConNF.ModelData α} {D₂ : ConNF.ModelData β} (h₁ : α = β) (h₂ : HEq D₁ D₂) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def ConNF.castTangle [ConNF.Params] {α β : ConNF.TypeIndex} {D₁ : ConNF.ModelData α} {D₂ : ConNF.ModelData β} (h₁ : α = β) (h₂ : HEq D₁ D₂) :
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              theorem ConNF.castTSet_forget [ConNF.Params] {α : ConNF.TypeIndex} {D₁ D₂ : ConNF.ModelData α} (h₂ : HEq D₁ D₂) (ρ : ConNF.TSet α) :
              theorem ConNF.castAllPerm_forget [ConNF.Params] {α : ConNF.TypeIndex} {D₁ D₂ : ConNF.ModelData α} (h₂ : HEq D₁ D₂) (ρ : ConNF.AllPerm α) :
              theorem ConNF.castTangle_support [ConNF.Params] {α : ConNF.TypeIndex} {D₁ D₂ : ConNF.ModelData α} (h₂ : HEq D₁ D₂) (t : ConNF.Tangle α) :
              ((ConNF.castTangle h₂) t).support = t.support
              theorem ConNF.castAllPerm_smul [ConNF.Params] {α : ConNF.TypeIndex} {D₁ D₂ : ConNF.ModelData α} (h₂ : HEq D₁ D₂) (ρ : ConNF.AllPerm α) (t : ConNF.Tangle α) :
              ρ (ConNF.castTangle h₂) t = (ConNF.castTangle h₂) ((ConNF.castAllPerm h₂).symm ρ t)
              theorem ConNF.castTangle_pos [ConNF.Params] {α β : ConNF.TypeIndex} {D₁ : ConNF.ModelData α} {D₂ : ConNF.ModelData β} {E₁ : ConNF.Position (ConNF.Tangle α)} {E₂ : ConNF.Position (ConNF.Tangle β)} (h₁ : α = β) (h₂ : HEq D₁ D₂) (h₃ : HEq E₁ E₂) (t : ConNF.Tangle α) :
              ConNF.pos ((ConNF.castTangle h₁ h₂) t) = ConNF.pos t
              theorem ConNF.castTangle_fuzz [ConNF.Params] {α : ConNF.TypeIndex} {D₁ D₂ : ConNF.ModelData α} {E₁ : ConNF.Position (ConNF.Tangle α)} {E₂ : ConNF.Position (ConNF.Tangle α)} (h₂ : HEq D₁ D₂) (h₃ : HEq E₁ E₂) (t : ConNF.Tangle α) {β : ConNF.Λ} (hαβ : α β) :
              ConNF.fuzz hαβ ((ConNF.castTangle h₂) t) = ConNF.fuzz hαβ t