We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
Condensed
1 parent 04c1c09 commit 983ee56Copy full SHA for 983ee56
Mathlib/Condensed/Basic.lean
@@ -37,14 +37,14 @@ open CategoryTheory Limits
37
38
open CategoryTheory
39
40
-universe u
+universe u v w
41
42
/--
43
`Condensed.{u} C` is the category of condensed objects in a category `C`, which are
44
defined as sheaves on `CompHaus.{u}` with respect to the coherent Grothendieck topology.
45
-/
46
-def Condensed (C : Type _) [Category C] :=
+def Condensed (C : Type w) [Category.{v} C] :=
47
Sheaf (coherentTopology CompHaus.{u}) C
48
49
-instance {C : Type _} [Category C] : Category (Condensed.{u} C) :=
+instance {C : Type w} [Category.{v} C] : Category (Condensed.{u} C) :=
50
show Category (Sheaf _ _) from inferInstance
0 commit comments