Documentation

ConNF.Structural.StructPerm

Structural permutations #

In this file, we define the ambient groups of structural permutations. These will later have recursively-constructed subgroups of allowable permutations which will act on t-sets; we define these larger ambient groups in advance in order to set up their infrastructure of derivatives and so on independently of the recursion.

We define structural permutations as trees of base permutations.

Main declarations #

@[reducible, inline]
abbrev ConNF.StructPerm [ConNF.Params] :
ConNF.TypeIndexType u

A structural permutation on a proper type index α is a base permutation for each α-extended index. This represents how the permutation acts along each path down the type levels in the model. Note that we define structural permutations as trees of near-litter permutations.

Equations
Instances For

    The following lemmas show how the action of -structural permutations on near-litters behaves; this is exactly how base permutations behave.

    @[simp]
    theorem ConNF.StructPerm.smul_nearLitter_fst [ConNF.Params] (π : ConNF.StructPerm ) (N : ConNF.NearLitter) :
    (π N).fst = π N.fst
    theorem ConNF.StructPerm.smul_nearLitter_coe [ConNF.Params] (π : ConNF.StructPerm ) (N : ConNF.NearLitter) :
    (π N) = π N
    theorem ConNF.StructPerm.smul_nearLitter_snd [ConNF.Params] (π : ConNF.StructPerm ) (N : ConNF.NearLitter) :
    (π N).snd = π N.snd
    @[simp]
    theorem ConNF.StructPerm.comp_bot_smul_atom [ConNF.Params] {α : ConNF.TypeIndex} (π : ConNF.StructPerm α) (A : ConNF.ExtendedIndex α) (a : ConNF.Atom) :
    ConNF.Tree.comp A π a = π A a
    @[simp]
    theorem ConNF.StructPerm.comp_bot_smul_litter [ConNF.Params] {α : ConNF.TypeIndex} (π : ConNF.StructPerm α) (A : ConNF.ExtendedIndex α) (L : ConNF.Litter) :
    ConNF.Tree.comp A π L = π A L
    @[simp]
    theorem ConNF.StructPerm.comp_bot_smul_nearLitter [ConNF.Params] {α : ConNF.TypeIndex} (π : ConNF.StructPerm α) (A : ConNF.ExtendedIndex α) (N : ConNF.NearLitter) :
    ConNF.Tree.comp A π N = π A N
    @[irreducible]
    Equations
    • One or more equations did not get rendered due to their size.
    • π.structSetAction t = ConNF.StructSet.toBot (ConNF.Tree.ofBot π ConNF.StructSet.ofBot t)
    Instances For
      theorem ConNF.StructPerm.mul_structSetAction [ConNF.Params] {α : ConNF.TypeIndex} (π₁ : ConNF.StructPerm α) (π₂ : ConNF.StructPerm α) (t : ConNF.StructSet α) :
      (π₁ * π₂).structSetAction t = π₁.structSetAction (π₂.structSetAction t)
      Equations
      theorem ConNF.StructPerm.smul_eq [ConNF.Params] {α : ConNF.TypeIndex} (π : ConNF.StructPerm α) (t : ConNF.StructSet α) :
      π t = π.structSetAction t
      theorem ConNF.StructPerm.smul_bot_eq [ConNF.Params] (π : ConNF.StructPerm ) (t : ConNF.StructSet ) :
      π t = ConNF.StructSet.toBot (ConNF.Tree.ofBot π ConNF.StructSet.ofBot t)
      theorem ConNF.StructPerm.ofCoe_smul [ConNF.Params] {α : ConNF.Λ} {β : ConNF.TypeIndex} (π : ConNF.StructPerm α) (t : ConNF.StructSet α) (h : β < α) :
      ConNF.StructSet.ofCoe (π t) β h = ConNF.Tree.comp (Quiver.Hom.toPath h) π ConNF.StructSet.ofCoe t β h