Skip to content

Commit 983ee56

Browse files
committed
chore: fix universe parameters in Condensed. (#5574)
1 parent 04c1c09 commit 983ee56

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

Mathlib/Condensed/Basic.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -37,14 +37,14 @@ open CategoryTheory Limits
3737

3838
open CategoryTheory
3939

40-
universe u
40+
universe u v w
4141

4242
/--
4343
`Condensed.{u} C` is the category of condensed objects in a category `C`, which are
4444
defined as sheaves on `CompHaus.{u}` with respect to the coherent Grothendieck topology.
4545
-/
46-
def Condensed (C : Type _) [Category C] :=
46+
def Condensed (C : Type w) [Category.{v} C] :=
4747
Sheaf (coherentTopology CompHaus.{u}) C
4848

49-
instance {C : Type _} [Category C] : Category (Condensed.{u} C) :=
49+
instance {C : Type w} [Category.{v} C] : Category (Condensed.{u} C) :=
5050
show Category (Sheaf _ _) from inferInstance

0 commit comments

Comments
 (0)