Zulip Chat Archive

Stream: maths

Topic: definition of sheaf of modules


Jujian Zhang (Dec 11 2021 at 15:55):

I am trying to write down a definition of (pre)sheaf of modules. I can think of two ways of doing this:

  1. be explicit about what the (pre)sheaf of ring is:
structure PresheafOfModules1 (X : Top) :=
(𝒪 : presheaf CommRing X)
( : presheaf AddCommGroup X)
[is_module : Π (U : (opens X)ᵒᵖ), module (𝒪.obj U) (ℱ.obj U)]
(res_compatible : Π (U V : (opens X)ᵒᵖ) (h : U  V) (r : 𝒪.obj U) (a: ℱ.obj U),
  ℱ.map h (r  a) = 𝒪.map h r  ℱ.map h a)
  1. be implicit about what the ring is:
class PresheafOfModules2 {X : Top} ( : @presheaf BundledModule BundledModule.is_cat X):=
(res_compatible :
  Π (U V : (opens X)ᵒᵖ) (h : U  V) (r : (ℱ.obj U).R) (m : (ℱ.obj U).M),
    (ℱ.map h).2 (r  m) = (r  (ℱ.map h).2 m))

Here bundled module is the category of pairs (R,M)(R, M) where RR is a ring and MM is an RR-module.

Which way, if any, is a good definition? Or is there a better way.

Johan Commelin (Dec 11 2021 at 15:56):

Did you see https://leanprover.zulipchat.com/#narrow/stream/267928-condensed-mathematics/topic/tensor.20product.20of.20sheaves/near/263012430?

Johan Commelin (Dec 11 2021 at 15:57):

(And the messages that follow it)

Jujian Zhang (Dec 11 2021 at 15:58):

I actually write restrict of scalars part and finished the bundled module category

Jujian Zhang (Dec 11 2021 at 15:58):

Could it be useful if I pr it, even if it didn't end up being used in defining sheaf of modules

Jujian Zhang (Dec 11 2021 at 16:00):

https://github.com/jjaassoonn/sheaf_of_modules

Kevin Buzzard (Dec 11 2021 at 16:01):

My guess is that nobody really knows which definition will be better, and we'll only find out once we start proving theorems about the idea.

Kevin Buzzard (Dec 11 2021 at 16:01):

My guess is that some stuff will be easier with one definition and some stuff will be easier with the other definition, and the real question will in some sense be whether the stuff which is easier with one definition is just completely horrible with the other definition, or whether it's not too bad.

Andrew Yang (Dec 11 2021 at 16:09):

Isn't the axiom in res_compatible part of the definition of what a hom in BundledModule is?

Jujian Zhang (Dec 11 2021 at 16:13):

Bundled module tells that r • (ℱ.map h).2 m) is actually (ℱ.map h).1 r • (ℱ.map h).2 m) but not saying that (ℱ.map h).2 (r • m) = (r • (ℱ.map h).2 m))

Andrew Yang (Dec 11 2021 at 16:23):

I may be missing something here, but given a map (f,f):(R,M)(S,N)(f, f') : (R, M) \to (S, N), the fact that f:MfNf' : M \to f^{*}N is a map of $R$-modules should tell you that f(rm)=rf(m)f'(r\cdot m) = r \cdot f'(m).

Jujian Zhang (Dec 11 2021 at 16:28):

You are absolutely right.

Adam Topaz (Dec 11 2021 at 16:28):

If you use the category you called BundledModule, you could just take presheaves resp. sheaves with values in that given category. I don't see why you need any further axioms. Then prove that the forgetful functor from that category to the category of rings preserves limits to obtain the forgetful functor from sheaves taking values in BundledModule to sheaves of rings.

Jujian Zhang (Dec 11 2021 at 16:29):

Yes.

Adam Topaz (Dec 11 2021 at 16:29):

docs#category_theory.Sheaf_compose

Jujian Zhang (Dec 11 2021 at 16:29):

Should I make a pr about bundledModule

Andrew Yang (Dec 11 2021 at 16:30):

I think this should be useful regardless of the final definition of sheaves of modules.

Jujian Zhang (Dec 11 2021 at 16:30):

Thank you. Sorry about the confusion. Let me pr bundled module

Kevin Buzzard (Dec 11 2021 at 16:31):

Note that linear_map is now precisely the morphism you want.

Kevin Buzzard (Dec 11 2021 at 16:31):

(I just read the most recent community blog post)

Jujian Zhang (Dec 11 2021 at 16:32):

I thought the explicit sheaf of ring definition is somewhat cumbersome exactly because the restriction map is just a map of abelian groups. But I forget that linear_map has map_smul

Adam Topaz (Dec 11 2021 at 16:34):

I think Kevin is referring to the fact that linear maps are now just a special case of a semilinear map

Andrew Yang (Dec 11 2021 at 16:35):

Regarding the definition of sheaves of modules, I would prefer the second one, especially after the recent advancements Adam has made in the sheaf library.

Kevin Buzzard (Dec 11 2021 at 16:35):

Adam: to my surprise, semilinear maps are now called linear_map.

Adam Topaz (Dec 11 2021 at 16:40):

@Jujian Zhang here is an approximation for how I would start the definition, with the new semilinear map stuff:

import algebra.category.Module.basic
import algebra.category.CommRing

universe u
structure BundledModule : Type (u+1) :=
(A : CommRing.{u})
(M : Module.{u} A)

structure BundledModule.hom (X Y : BundledModule) :=
(f : X.A  Y.A)
(g : X.M →ₛₗ[f] Y.M)

Adam Topaz (Dec 11 2021 at 16:40):

(I don't know whether you already have a definition of BundledModule)

Adam Topaz (Dec 11 2021 at 16:45):

You could generalize the universe levels, but I don't know how useful that would be.

Kevin Buzzard (Dec 11 2021 at 17:05):

I'll remark that Jujian and I have already discussed this issue a bit, and at some point he was having trouble with universes, and I already suggested that he used fewer than 4 :-)


Last updated: Dec 20 2023 at 11:08 UTC