Skip to content

Commit

Permalink
style: pp_with_univ for TypeVec & PFunctor & MvPFunctor (#7742)
Browse files Browse the repository at this point in the history
  • Loading branch information
Komyyy committed Oct 18, 2023
1 parent 5cff8eb commit 68b12e1
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Data/PFunctor/Multivariate/Basic.lean
Expand Up @@ -24,6 +24,7 @@ open MvFunctor

/-- multivariate polynomial functors
-/
@[pp_with_univ]
structure MvPFunctor (n : ℕ) where
/-- The head type -/
A : Type u
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Data/PFunctor/Univariate/Basic.lean
Expand Up @@ -27,6 +27,7 @@ An element of `P.obj α` is a pair `⟨a, f⟩`, where `a` is an element of a ty
`f : B a → α`. Think of `a` as the shape of the object and `f` as an index to the relevant
elements of `α`.
-/
@[pp_with_univ]
structure PFunctor where
/-- The head type -/
A : Type u
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Data/TypeVec.lean
Expand Up @@ -35,6 +35,7 @@ to it, we need support functions and lemmas to mediate between constructions.
universe u v w

/-- n-tuples of types, as a category -/
@[pp_with_univ]
def TypeVec (n : ℕ) :=
Fin2 n → Type*
#align typevec TypeVec
Expand Down

0 comments on commit 68b12e1

Please sign in to comment.