Documentation

Mathlib.Data.TypeVec

Tuples of types, and their categorical structure. #

Features #

Also, support functions for operating with n-tuples of types, such as:

Since e.g. append1 α.drop α.last is propositionally equal to α but not definitionally equal to it, we need support functions and lemmas to mediate between constructions.

def TypeVec (n : ) :
Type (u_1 + 1)

n-tuples of types, as a category

Equations
Instances For
    Equations
    def TypeVec.Arrow {n : } (α : TypeVec.{u_1} n) (β : TypeVec.{u_2} n) :
    Type (max u_1 u_2)

    arrow in the category of TypeVec

    Equations
    Instances For
      theorem TypeVec.Arrow.ext {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_2} n} (f : TypeVec.Arrow α β) (g : TypeVec.Arrow α β) :
      (∀ (i : Fin2 n), f i = g i)f = g

      Extensionality for arrows

      instance TypeVec.Arrow.inhabited {n : } (α : TypeVec.{u_1} n) (β : TypeVec.{u_2} n) [(i : Fin2 n) → Inhabited (β i)] :
      Equations
      def TypeVec.id {n : } {α : TypeVec.{u_1} n} :

      identity of arrow composition

      Equations
      Instances For
        def TypeVec.comp {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_2} n} {γ : TypeVec.{u_3} n} (g : TypeVec.Arrow β γ) (f : TypeVec.Arrow α β) :

        arrow composition in the category of TypeVec

        Equations
        Instances For

          arrow composition in the category of TypeVec

          Equations
          Instances For
            @[simp]
            theorem TypeVec.id_comp {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_2} n} (f : TypeVec.Arrow α β) :
            TypeVec.comp TypeVec.id f = f
            @[simp]
            theorem TypeVec.comp_id {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_2} n} (f : TypeVec.Arrow α β) :
            TypeVec.comp f TypeVec.id = f
            theorem TypeVec.comp_assoc {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_2} n} {γ : TypeVec.{u_3} n} {δ : TypeVec.{u_4} n} (h : TypeVec.Arrow γ δ) (g : TypeVec.Arrow β γ) (f : TypeVec.Arrow α β) :
            def TypeVec.append1 {n : } (α : TypeVec.{u_1} n) (β : Type u_1) :

            Support for extending a TypeVec by one element.

            Equations
            • (α ::: β) x = match x with | Fin2.fs i => α i | Fin2.fz => β
            Instances For

              Support for extending a TypeVec by one element.

              Equations
              Instances For
                def TypeVec.drop {n : } (α : TypeVec.{u} (n + 1)) :

                retain only a n-length prefix of the argument

                Equations
                Instances For
                  def TypeVec.last {n : } (α : TypeVec.{u} (n + 1)) :

                  take the last value of a (n+1)-length vector

                  Equations
                  Instances For
                    instance TypeVec.last.inhabited {n : } (α : TypeVec.{u_1} (n + 1)) [Inhabited (α Fin2.fz)] :
                    Equations
                    theorem TypeVec.drop_append1 {n : } {α : TypeVec.{u_1} n} {β : Type u_1} {i : Fin2 n} :
                    TypeVec.drop (α ::: β) i = α i
                    @[simp]
                    theorem TypeVec.drop_append1' {n : } {α : TypeVec.{u_1} n} {β : Type u_1} :
                    TypeVec.drop (α ::: β) = α
                    theorem TypeVec.last_append1 {n : } {α : TypeVec.{u_1} n} {β : Type u_1} :
                    TypeVec.last (α ::: β) = β
                    @[simp]
                    def TypeVec.append1Cases {n : } {C : TypeVec.{u_1} (n + 1)Sort u} (H : (α : TypeVec.{u_1} n) → (β : Type u_1) → C (α ::: β)) (γ : TypeVec.{u_1} (n + 1)) :
                    C γ

                    cases on (n+1)-length vectors

                    Equations
                    Instances For
                      @[simp]
                      theorem TypeVec.append1_cases_append1 {n : } {C : TypeVec.{u_1} (n + 1)Sort u} (H : (α : TypeVec.{u_1} n) → (β : Type u_1) → C (α ::: β)) (α : TypeVec.{u_1} n) (β : Type u_1) :
                      TypeVec.append1Cases H (α ::: β) = H α β
                      def TypeVec.splitFun {n : } {α : TypeVec.{u_1} (n + 1)} {α' : TypeVec.{u_2} (n + 1)} (f : TypeVec.Arrow (TypeVec.drop α) (TypeVec.drop α')) (g : TypeVec.last αTypeVec.last α') :

                      append an arrow and a function for arbitrary source and target type vectors

                      Equations
                      Instances For
                        def TypeVec.appendFun {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_2} n} {β : Type u_1} {β' : Type u_2} (f : TypeVec.Arrow α α') (g : ββ') :
                        TypeVec.Arrow (α ::: β) (α' ::: β')

                        append an arrow and a function as well as their respective source and target types / typevecs

                        Equations
                        Instances For

                          append an arrow and a function as well as their respective source and target types / typevecs

                          Equations
                          Instances For
                            def TypeVec.dropFun {n : } {α : TypeVec.{u_1} (n + 1)} {β : TypeVec.{u_2} (n + 1)} (f : TypeVec.Arrow α β) :

                            split off the prefix of an arrow

                            Equations
                            Instances For
                              def TypeVec.lastFun {n : } {α : TypeVec.{u_1} (n + 1)} {β : TypeVec.{u_2} (n + 1)} (f : TypeVec.Arrow α β) :

                              split off the last function of an arrow

                              Equations
                              Instances For

                                arrow in the category of 0-length vectors

                                Equations
                                Instances For
                                  theorem TypeVec.eq_of_drop_last_eq {n : } {α : TypeVec.{u_1} (n + 1)} {β : TypeVec.{u_2} (n + 1)} {f : TypeVec.Arrow α β} {g : TypeVec.Arrow α β} (h₀ : TypeVec.dropFun f = TypeVec.dropFun g) (h₁ : TypeVec.lastFun f = TypeVec.lastFun g) :
                                  f = g
                                  @[simp]
                                  def TypeVec.Arrow.mp {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} (h : α = β) :

                                  turn an equality into an arrow

                                  Equations
                                  Instances For
                                    def TypeVec.Arrow.mpr {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} (h : α = β) :

                                    turn an equality into an arrow, with reverse direction

                                    Equations
                                    Instances For

                                      decompose a vector into its prefix appended with its last element

                                      Equations
                                      Instances For

                                        stitch two bits of a vector back together

                                        Equations
                                        Instances For
                                          @[simp]
                                          @[simp]
                                          theorem TypeVec.dropFun_appendFun {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_2} n} {β : Type u_1} {β' : Type u_2} (f : TypeVec.Arrow α α') (g : ββ') :
                                          @[simp]
                                          theorem TypeVec.lastFun_appendFun {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_2} n} {β : Type u_1} {β' : Type u_2} (f : TypeVec.Arrow α α') (g : ββ') :
                                          theorem TypeVec.splitFun_inj {n : } {α : TypeVec.{u_1} (n + 1)} {α' : TypeVec.{u_2} (n + 1)} {f : TypeVec.Arrow (TypeVec.drop α) (TypeVec.drop α')} {f' : TypeVec.Arrow (TypeVec.drop α) (TypeVec.drop α')} {g : TypeVec.last αTypeVec.last α'} {g' : TypeVec.last αTypeVec.last α'} (H : TypeVec.splitFun f g = TypeVec.splitFun f' g') :
                                          f = f' g = g'
                                          theorem TypeVec.appendFun_inj {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_2} n} {β : Type u_1} {β' : Type u_2} {f : TypeVec.Arrow α α'} {f' : TypeVec.Arrow α α'} {g : ββ'} {g' : ββ'} :
                                          (f ::: g) = (f' ::: g')f = f' g = g'
                                          theorem TypeVec.splitFun_comp {n : } {α₀ : TypeVec.{u_1} (n + 1)} {α₁ : TypeVec.{u_2} (n + 1)} {α₂ : TypeVec.{u_3} (n + 1)} (f₀ : TypeVec.Arrow (TypeVec.drop α₀) (TypeVec.drop α₁)) (f₁ : TypeVec.Arrow (TypeVec.drop α₁) (TypeVec.drop α₂)) (g₀ : TypeVec.last α₀TypeVec.last α₁) (g₁ : TypeVec.last α₁TypeVec.last α₂) :
                                          TypeVec.splitFun (TypeVec.comp f₁ f₀) (g₁ g₀) = TypeVec.comp (TypeVec.splitFun f₁ g₁) (TypeVec.splitFun f₀ g₀)
                                          theorem TypeVec.appendFun_comp_splitFun {n : } {α : TypeVec.{u_1} n} {γ : TypeVec.{u_2} n} {β : Type u_1} {δ : Type u_2} {ε : TypeVec.{u_3} (n + 1)} (f₀ : TypeVec.Arrow (TypeVec.drop ε) α) (f₁ : TypeVec.Arrow α γ) (g₀ : TypeVec.last εβ) (g₁ : βδ) :
                                          TypeVec.comp (f₁ ::: g₁) (TypeVec.splitFun f₀ g₀) = TypeVec.splitFun (TypeVec.comp f₁ f₀) (g₁ g₀)
                                          theorem TypeVec.appendFun_comp {n : } {α₀ : TypeVec.{u_1} n} {α₁ : TypeVec.{u_2} n} {α₂ : TypeVec.{u_3} n} {β₀ : Type u_1} {β₁ : Type u_2} {β₂ : Type u_3} (f₀ : TypeVec.Arrow α₀ α₁) (f₁ : TypeVec.Arrow α₁ α₂) (g₀ : β₀β₁) (g₁ : β₁β₂) :
                                          (TypeVec.comp f₁ f₀ ::: g₁ g₀) = TypeVec.comp (f₁ ::: g₁) (f₀ ::: g₀)
                                          theorem TypeVec.appendFun_comp' {n : } {α₀ : TypeVec.{u_1} n} {α₁ : TypeVec.{u_2} n} {α₂ : TypeVec.{u_3} n} {β₀ : Type u_1} {β₁ : Type u_2} {β₂ : Type u_3} (f₀ : TypeVec.Arrow α₀ α₁) (f₁ : TypeVec.Arrow α₁ α₂) (g₀ : β₀β₁) (g₁ : β₁β₂) :
                                          TypeVec.comp (f₁ ::: g₁) (f₀ ::: g₀) = (TypeVec.comp f₁ f₀ ::: g₁ g₀)
                                          theorem TypeVec.nilFun_comp {α₀ : TypeVec.{u_1} 0} (f₀ : TypeVec.Arrow α₀ Fin2.elim0) :
                                          TypeVec.comp TypeVec.nilFun f₀ = f₀
                                          theorem TypeVec.appendFun_comp_id {n : } {α : TypeVec.{u} n} {β₀ : Type u} {β₁ : Type u} {β₂ : Type u} (g₀ : β₀β₁) (g₁ : β₁β₂) :
                                          (TypeVec.id ::: g₁ g₀) = TypeVec.comp (TypeVec.id ::: g₁) (TypeVec.id ::: g₀)
                                          @[simp]
                                          theorem TypeVec.dropFun_comp {n : } {α₀ : TypeVec.{u_1} (n + 1)} {α₁ : TypeVec.{u_2} (n + 1)} {α₂ : TypeVec.{u_3} (n + 1)} (f₀ : TypeVec.Arrow α₀ α₁) (f₁ : TypeVec.Arrow α₁ α₂) :
                                          @[simp]
                                          theorem TypeVec.lastFun_comp {n : } {α₀ : TypeVec.{u_1} (n + 1)} {α₁ : TypeVec.{u_2} (n + 1)} {α₂ : TypeVec.{u_3} (n + 1)} (f₀ : TypeVec.Arrow α₀ α₁) (f₁ : TypeVec.Arrow α₁ α₂) :
                                          theorem TypeVec.appendFun_aux {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_2} n} {β : Type u_1} {β' : Type u_2} (f : TypeVec.Arrow (α ::: β) (α' ::: β')) :
                                          theorem TypeVec.appendFun_id_id {n : } {α : TypeVec.{u_1} n} {β : Type u_1} :
                                          (TypeVec.id ::: id) = TypeVec.id
                                          def TypeVec.casesNil {β : TypeVec.{u_2} 0Sort u_1} (f : β Fin2.elim0) (v : TypeVec.{u_2} 0) :
                                          β v

                                          cases distinction for 0-length type vector

                                          Equations
                                          Instances For
                                            def TypeVec.casesCons (n : ) {β : TypeVec.{u_2} (n + 1)Sort u_1} (f : (t : Type u_2) → (v : TypeVec.{u_2} n) → β (v ::: t)) (v : TypeVec.{u_2} (n + 1)) :
                                            β v

                                            cases distinction for (n+1)-length type vector

                                            Equations
                                            Instances For
                                              theorem TypeVec.casesNil_append1 {β : TypeVec.{u_2} 0Sort u_1} (f : β Fin2.elim0) :
                                              TypeVec.casesNil f Fin2.elim0 = f
                                              theorem TypeVec.casesCons_append1 (n : ) {β : TypeVec.{u_2} (n + 1)Sort u_1} (f : (t : Type u_2) → (v : TypeVec.{u_2} n) → β (v ::: t)) (v : TypeVec.{u_2} n) (α : Type u_2) :
                                              TypeVec.casesCons n f (v ::: α) = f α v
                                              def TypeVec.typevecCasesNil₃ {β : (v : TypeVec.{u_2} 0) → (v' : TypeVec.{u_3} 0) → TypeVec.Arrow v v'Sort u_1} (f : β Fin2.elim0 Fin2.elim0 TypeVec.nilFun) (v : TypeVec.{u_2} 0) (v' : TypeVec.{u_3} 0) (fs : TypeVec.Arrow v v') :
                                              β v v' fs

                                              cases distinction for an arrow in the category of 0-length type vectors

                                              Equations
                                              Instances For
                                                def TypeVec.typevecCasesCons₃ (n : ) {β : (v : TypeVec.{u_2} (n + 1)) → (v' : TypeVec.{u_3} (n + 1)) → TypeVec.Arrow v v'Sort u_1} (F : (t : Type u_2) → (t' : Type u_3) → (f : tt') → (v : TypeVec.{u_2} n) → (v' : TypeVec.{u_3} n) → (fs : TypeVec.Arrow v v') → β (v ::: t) (v' ::: t') (fs ::: f)) (v : TypeVec.{u_2} (n + 1)) (v' : TypeVec.{u_3} (n + 1)) (fs : TypeVec.Arrow v v') :
                                                β v v' fs

                                                cases distinction for an arrow in the category of (n+1)-length type vectors

                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                Instances For
                                                  def TypeVec.typevecCasesNil₂ {β : TypeVec.Arrow Fin2.elim0 Fin2.elim0Sort u_1} (f : β TypeVec.nilFun) (f : TypeVec.Arrow Fin2.elim0 Fin2.elim0) :
                                                  β f

                                                  specialized cases distinction for an arrow in the category of 0-length type vectors

                                                  Equations
                                                  Instances For
                                                    def TypeVec.typevecCasesCons₂ (n : ) (t : Type u_1) (t' : Type u_2) (v : TypeVec.{u_1} n) (v' : TypeVec.{u_2} n) {β : TypeVec.Arrow (v ::: t) (v' ::: t')Sort u_3} (F : (f : tt') → (fs : TypeVec.Arrow v v') → β (fs ::: f)) (fs : TypeVec.Arrow (v ::: t) (v' ::: t')) :
                                                    β fs

                                                    specialized cases distinction for an arrow in the category of (n+1)-length type vectors

                                                    Equations
                                                    Instances For
                                                      theorem TypeVec.typevecCasesNil₂_appendFun {β : TypeVec.Arrow Fin2.elim0 Fin2.elim0Sort u_1} (f : β TypeVec.nilFun) :
                                                      TypeVec.typevecCasesNil₂ f TypeVec.nilFun = f
                                                      theorem TypeVec.typevecCasesCons₂_appendFun (n : ) (t : Type u_1) (t' : Type u_2) (v : TypeVec.{u_1} n) (v' : TypeVec.{u_2} n) {β : TypeVec.Arrow (v ::: t) (v' ::: t')Sort u_3} (F : (f : tt') → (fs : TypeVec.Arrow v v') → β (fs ::: f)) (f : tt') (fs : TypeVec.Arrow v v') :
                                                      TypeVec.typevecCasesCons₂ n t t' v v' F (fs ::: f) = F f fs
                                                      def TypeVec.PredLast {n : } (α : TypeVec.{u_1} n) {β : Type u_1} (p : βProp) ⦃i : Fin2 (n + 1) :
                                                      (α ::: β) iProp

                                                      PredLast α p x predicates p of the last element of x : α.append1 β.

                                                      Equations
                                                      Instances For
                                                        def TypeVec.RelLast {n : } (α : TypeVec.{u} n) {β : Type u} {γ : Type u} (r : βγProp) ⦃i : Fin2 (n + 1) :
                                                        (α ::: β) i(α ::: γ) iProp

                                                        RelLast α r x y says that p the last elements of x y : α.append1 β are related by r and all the other elements are equal.

                                                        Equations
                                                        Instances For
                                                          def TypeVec.repeat (n : ) :

                                                          repeat n t is a n-length type vector that contains n occurrences of t

                                                          Equations
                                                          Instances For

                                                            prod α β is the pointwise product of the components of α and β

                                                            Equations
                                                            Instances For

                                                              prod α β is the pointwise product of the components of α and β

                                                              Equations
                                                              Instances For
                                                                def TypeVec.const {β : Type u_1} (x : β) {n : } (α : TypeVec.{u_2} n) :

                                                                const x α is an arrow that ignores its source and constructs a TypeVec that contains nothing but x

                                                                Equations
                                                                Instances For

                                                                  vector of equality on a product of vectors

                                                                  Equations
                                                                  Instances For
                                                                    theorem TypeVec.const_append1 {β : Type u_1} {γ : Type u_2} (x : γ) {n : } (α : TypeVec.{u_1} n) :
                                                                    TypeVec.const x (α ::: β) = (TypeVec.const x α ::: fun (x_1 : β) => x)
                                                                    theorem TypeVec.eq_nilFun {α : TypeVec.{u_1} 0} {β : TypeVec.{u_2} 0} (f : TypeVec.Arrow α β) :
                                                                    f = TypeVec.nilFun
                                                                    theorem TypeVec.id_eq_nilFun {α : TypeVec.{u_1} 0} :
                                                                    TypeVec.id = TypeVec.nilFun
                                                                    theorem TypeVec.const_nil {β : Type u_1} (x : β) (α : TypeVec.{u_2} 0) :
                                                                    TypeVec.const x α = TypeVec.nilFun
                                                                    theorem TypeVec.repeat_eq_nil (α : TypeVec.{u_1} 0) :
                                                                    TypeVec.repeatEq α = TypeVec.nilFun
                                                                    def TypeVec.PredLast' {n : } (α : TypeVec.{u_1} n) {β : Type u_1} (p : βProp) :

                                                                    predicate on a type vector to constrain only the last object

                                                                    Equations
                                                                    Instances For
                                                                      def TypeVec.RelLast' {n : } (α : TypeVec.{u_1} n) {β : Type u_1} (p : ββProp) :

                                                                      predicate on the product of two type vectors to constrain only their last object

                                                                      Equations
                                                                      Instances For
                                                                        def TypeVec.Curry {n : } (F : TypeVec.{u} (n + 1)Type u_1) (α : Type u) (β : TypeVec.{u} n) :
                                                                        Type u_1

                                                                        given F : TypeVec.{u} (n+1) → Type u, curry F : Type u → TypeVec.{u} → Type u, i.e. its first argument can be fed in separately from the rest of the vector of arguments

                                                                        Equations
                                                                        Instances For
                                                                          instance TypeVec.Curry.inhabited {n : } (F : TypeVec.{u} (n + 1)Type u_1) (α : Type u) (β : TypeVec.{u} n) [I : Inhabited (F (β ::: α))] :
                                                                          Equations

                                                                          arrow to remove one element of a repeat vector

                                                                          Equations
                                                                          Instances For
                                                                            def TypeVec.ofRepeat {α : Type u_1} {n : } {i : Fin2 n} :
                                                                            TypeVec.repeat n α iα

                                                                            projection for a repeat vector

                                                                            Equations
                                                                            • TypeVec.ofRepeat = fun (a : α) => a
                                                                            • TypeVec.ofRepeat = TypeVec.ofRepeat
                                                                            Instances For
                                                                              theorem TypeVec.const_iff_true {n : } {α : TypeVec.{u_1} n} {i : Fin2 n} {x : α i} {p : Prop} :
                                                                              def TypeVec.prod.fst {n : } {α : TypeVec.{u} n} {β : TypeVec.{u} n} :

                                                                              left projection of a prod vector

                                                                              Equations
                                                                              Instances For
                                                                                def TypeVec.prod.snd {n : } {α : TypeVec.{u} n} {β : TypeVec.{u} n} :

                                                                                right projection of a prod vector

                                                                                Equations
                                                                                Instances For

                                                                                  introduce a product where both components are the same

                                                                                  Equations
                                                                                  Instances For
                                                                                    def TypeVec.prod.mk {n : } {α : TypeVec.{u} n} {β : TypeVec.{u} n} (i : Fin2 n) :
                                                                                    α iβ iTypeVec.prod α β i

                                                                                    constructor for prod

                                                                                    Equations
                                                                                    Instances For
                                                                                      @[simp]
                                                                                      theorem TypeVec.prod_fst_mk {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} (i : Fin2 n) (a : α i) (b : β i) :
                                                                                      @[simp]
                                                                                      theorem TypeVec.prod_snd_mk {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} (i : Fin2 n) (a : α i) (b : β i) :
                                                                                      def TypeVec.prod.map {n : } {α : TypeVec.{u} n} {α' : TypeVec.{u} n} {β : TypeVec.{u} n} {β' : TypeVec.{u} n} :
                                                                                      TypeVec.Arrow α βTypeVec.Arrow α' β'TypeVec.Arrow (TypeVec.prod α α') (TypeVec.prod β β')

                                                                                      prod is functorial

                                                                                      Equations
                                                                                      Instances For
                                                                                        theorem TypeVec.fst_prod_mk {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} {β' : TypeVec.{u_1} n} (f : TypeVec.Arrow α β) (g : TypeVec.Arrow α' β') :
                                                                                        TypeVec.comp TypeVec.prod.fst (TypeVec.prod.map f g) = TypeVec.comp f TypeVec.prod.fst
                                                                                        theorem TypeVec.snd_prod_mk {n : } {α : TypeVec.{u_1} n} {α' : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} {β' : TypeVec.{u_1} n} (f : TypeVec.Arrow α β) (g : TypeVec.Arrow α' β') :
                                                                                        TypeVec.comp TypeVec.prod.snd (TypeVec.prod.map f g) = TypeVec.comp g TypeVec.prod.snd
                                                                                        theorem TypeVec.fst_diag {n : } {α : TypeVec.{u_1} n} :
                                                                                        TypeVec.comp TypeVec.prod.fst TypeVec.prod.diag = TypeVec.id
                                                                                        theorem TypeVec.snd_diag {n : } {α : TypeVec.{u_1} n} :
                                                                                        TypeVec.comp TypeVec.prod.snd TypeVec.prod.diag = TypeVec.id
                                                                                        theorem TypeVec.repeatEq_iff_eq {n : } {α : TypeVec.{u_1} n} {i : Fin2 n} {x : α i} {y : α i} :

                                                                                        given a predicate vector p over vector α, Subtype_ p is the type of vectors that contain an α that satisfies p

                                                                                        Equations
                                                                                        Instances For

                                                                                          projection on Subtype_

                                                                                          Equations
                                                                                          Instances For
                                                                                            def TypeVec.toSubtype {n : } {α : TypeVec.{u} n} (p : TypeVec.Arrow α (TypeVec.repeat n Prop)) :
                                                                                            TypeVec.Arrow (fun (i : Fin2 n) => { x : α i // TypeVec.ofRepeat (p i x) }) (TypeVec.Subtype_ p)

                                                                                            arrow that rearranges the type of Subtype_ to turn a subtype of vector into a vector of subtypes

                                                                                            Equations
                                                                                            Instances For
                                                                                              def TypeVec.ofSubtype {n : } {α : TypeVec.{u} n} (p : TypeVec.Arrow α (TypeVec.repeat n Prop)) :
                                                                                              TypeVec.Arrow (TypeVec.Subtype_ p) fun (i : Fin2 n) => { x : α i // TypeVec.ofRepeat (p i x) }

                                                                                              arrow that rearranges the type of Subtype_ to turn a vector of subtypes into a subtype of vector

                                                                                              Equations
                                                                                              Instances For
                                                                                                def TypeVec.toSubtype' {n : } {α : TypeVec.{u} n} (p : TypeVec.Arrow (TypeVec.prod α α) (TypeVec.repeat n Prop)) :
                                                                                                TypeVec.Arrow (fun (i : Fin2 n) => { x : α i × α i // TypeVec.ofRepeat (p i (TypeVec.prod.mk i x.1 x.2)) }) (TypeVec.Subtype_ p)

                                                                                                similar to toSubtype adapted to relations (i.e. predicate on product)

                                                                                                Equations
                                                                                                Instances For
                                                                                                  def TypeVec.ofSubtype' {n : } {α : TypeVec.{u} n} (p : TypeVec.Arrow (TypeVec.prod α α) (TypeVec.repeat n Prop)) :
                                                                                                  TypeVec.Arrow (TypeVec.Subtype_ p) fun (i : Fin2 n) => { x : α i × α i // TypeVec.ofRepeat (p i (TypeVec.prod.mk i x.1 x.2)) }

                                                                                                  similar to of_subtype adapted to relations (i.e. predicate on product)

                                                                                                  Equations
                                                                                                  Instances For

                                                                                                    similar to diag but the target vector is a Subtype_ guaranteeing the equality of the components

                                                                                                    Equations
                                                                                                    Instances For
                                                                                                      theorem TypeVec.diag_sub_val {n : } {α : TypeVec.{u} n} :
                                                                                                      TypeVec.comp (TypeVec.subtypeVal (TypeVec.repeatEq α)) TypeVec.diagSub = TypeVec.prod.diag
                                                                                                      theorem TypeVec.prod_id {n : } {α : TypeVec.{u} n} {β : TypeVec.{u} n} :
                                                                                                      TypeVec.prod.map TypeVec.id TypeVec.id = TypeVec.id
                                                                                                      theorem TypeVec.append_prod_appendFun {n : } {α : TypeVec.{u} n} {α' : TypeVec.{u} n} {β : TypeVec.{u} n} {β' : TypeVec.{u} n} {φ : Type u} {φ' : Type u} {ψ : Type u} {ψ' : Type u} {f₀ : TypeVec.Arrow α α'} {g₀ : TypeVec.Arrow β β'} {f₁ : φφ'} {g₁ : ψψ'} :
                                                                                                      (TypeVec.prod.map f₀ g₀ ::: Prod.map f₁ g₁) = TypeVec.prod.map (f₀ ::: f₁) (g₀ ::: g₁)
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.dropFun_diag {n : } {α : TypeVec.{u_1} (n + 1)} :
                                                                                                      TypeVec.dropFun TypeVec.prod.diag = TypeVec.prod.diag
                                                                                                      @[simp]
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.dropFun_toSubtype {n : } {α : TypeVec.{u_1} (n + 1)} (p : TypeVec.Arrow α (TypeVec.repeat (n + 1) Prop)) :
                                                                                                      TypeVec.dropFun (TypeVec.toSubtype p) = TypeVec.toSubtype fun (i : Fin2 n) (x : α (Fin2.fs i)) => p (Fin2.fs i) x
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.dropFun_RelLast' {n : } {α : TypeVec.{u_1} n} {β : Type u_1} (R : ββProp) :
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.dropFun_prod {n : } {α : TypeVec.{u_1} (n + 1)} {α' : TypeVec.{u_1} (n + 1)} {β : TypeVec.{u_1} (n + 1)} {β' : TypeVec.{u_1} (n + 1)} (f : TypeVec.Arrow α β) (f' : TypeVec.Arrow α' β') :
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.lastFun_prod {n : } {α : TypeVec.{u_1} (n + 1)} {α' : TypeVec.{u_1} (n + 1)} {β : TypeVec.{u_1} (n + 1)} {β' : TypeVec.{u_1} (n + 1)} (f : TypeVec.Arrow α β) (f' : TypeVec.Arrow α' β') :
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.dropFun_from_append1_drop_last {n : } {α : TypeVec.{u_1} (n + 1)} :
                                                                                                      TypeVec.dropFun TypeVec.fromAppend1DropLast = TypeVec.id
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.lastFun_from_append1_drop_last {n : } {α : TypeVec.{u_1} (n + 1)} :
                                                                                                      TypeVec.lastFun TypeVec.fromAppend1DropLast = id
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.dropFun_id {n : } {α : TypeVec.{u_1} (n + 1)} :
                                                                                                      TypeVec.dropFun TypeVec.id = TypeVec.id
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.prod_map_id {n : } {α : TypeVec.{u_1} n} {β : TypeVec.{u_1} n} :
                                                                                                      TypeVec.prod.map TypeVec.id TypeVec.id = TypeVec.id
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.subtypeVal_diagSub {n : } {α : TypeVec.{u_1} n} :
                                                                                                      TypeVec.comp (TypeVec.subtypeVal (TypeVec.repeatEq α)) TypeVec.diagSub = TypeVec.prod.diag
                                                                                                      @[simp]
                                                                                                      theorem TypeVec.subtypeVal_toSubtype' {n : } {α : TypeVec.{u_1} n} (r : TypeVec.Arrow (TypeVec.prod α α) (TypeVec.repeat n Prop)) :
                                                                                                      TypeVec.comp (TypeVec.subtypeVal r) (TypeVec.toSubtype' r) = fun (i : Fin2 n) (x : (fun (i : Fin2 n) => { x : α i × α i // TypeVec.ofRepeat (r i (TypeVec.prod.mk i x.1 x.2)) }) i) => TypeVec.prod.mk i (x).1 (x).2