Skip to content

Commit

Permalink
Messed up vars order...
Browse files Browse the repository at this point in the history
  • Loading branch information
robin-carlier committed Feb 25, 2025
1 parent 90c6369 commit 3397ed2
Showing 1 changed file with 4 additions and 2 deletions.
6 changes: 4 additions & 2 deletions Mathlib/CategoryTheory/Sums/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -148,8 +148,10 @@ end Swap

end Sum

variable {A : Type u₁} [Category.{v₁} A] {B : Type u₂} [Category.{v₂} B] {C : Type u₁}
[Category.{v₁} C] {D : Type u₂} [Category.{v₂} D] {A' : Type u₁} [Category.{v₁} A']
variable {A : Type u₁} [Category.{v₁} A] {A' : Type u₁} [Category.{v₁} A']
{B : Type u₂} [Category.{v₂} B]
{C : Type u₁} [Category.{v₁} C]
{D : Type u₂} [Category.{v₂} D]

namespace Functor

Expand Down

0 comments on commit 3397ed2

Please sign in to comment.