Zulip Chat Archive

Stream: Is there code for X?

Topic: Canonical injection into the localization


Yaël Dillies (Apr 04 2023 at 17:36):

What is the idiomatic way to spell the canonical injection from a cancellative commutative monoid α to its localization localization s at a submonoid s? I'm really confused reading file#group_theory/monoid_localization.

Eric Rodriguez (Apr 04 2023 at 17:51):

I mean, it's not always injective

Yaël Dillies (Apr 04 2023 at 17:54):

Edited the crucial word in

Adam Topaz (Apr 04 2023 at 19:28):

Isn’t it just docs#localization_map ?

Adam Topaz (Apr 04 2023 at 19:29):

Modulo namespaces

Adam Topaz (Apr 04 2023 at 19:30):

If you use rings, then it would be an algebra_map but it seems you want to localize multiplicative monoids?

Adam Topaz (Apr 04 2023 at 19:33):

Btw I think it can be noninjective even for cancellative monoids

Yaël Dillies (Apr 04 2023 at 19:56):

Too bad, I proved it was injective in #18724!

Yaël Dillies (Apr 04 2023 at 19:57):

It's also "just" docs#localization.monoid_of or "just" docs#localization.mk. What I don't know is what's preferred.

Adam Topaz (Apr 04 2023 at 19:59):

Too bad. You didn’t say commutative in your original post.

Yaël Dillies (Apr 04 2023 at 20:00):

The correct amount of qualifiers should be inferred from the context :sweat_smile:

Yaël Dillies (Apr 04 2023 at 20:01):

For my defence, the entire file is about commutative monoids.

Adam Topaz (Apr 04 2023 at 20:07):

@Yaël Dillies in case you're curious: https://link.springer.com/article/10.1007/BF01571659

Adam Topaz (Apr 04 2023 at 20:08):

so are you saying that we can't localize noncommutative monoids (with current mathlib)?

Yaël Dillies (Apr 04 2023 at 20:09):

Indeed, that's my understanding.

Johan Commelin (Apr 04 2023 at 20:09):

We have Ore localizations, I think

Yaël Dillies (Apr 04 2023 at 20:10):

Oh right! I know nothing of those.

Yaël Dillies (Apr 04 2023 at 20:10):

... not that I care, because my result (#18724) only holds for commutative semigroups.

Johan Commelin (Apr 04 2023 at 20:10):

src/ring_theory/ore_localization/basic.lean

Eric Wieser (Apr 04 2023 at 20:55):

Do the notions coincide in the commutative case?

Riccardo Brasca (Apr 04 2023 at 23:32):

Eric Wieser said:

Do the notions coincide in the commutative case?

Yep

Reid Barton (Apr 05 2023 at 04:24):

semigroups? I'm confused

Reid Barton (Apr 05 2023 at 04:25):

Looking at the PR it doesn't use semigroups, so now I am less confused.

Reid Barton (Apr 05 2023 at 04:26):

BTW Ore localizations also exist for monoids even though they are in the ring_theory subdirectory for some reason--it's calculus of fractions stuff.

Yaël Dillies (Apr 05 2023 at 06:40):

Yeah, my result holds for nonempty semigroups but I can't state it as such with current mathlib.

Reid Barton (Apr 05 2023 at 06:56):

I think the empty semigroup also embeds in an ordered group. :upside_down:

Yaël Dillies (Apr 05 2023 at 06:58):

Yeah, but its Grothendieck group isn't a group!

Reid Barton (Apr 05 2023 at 07:07):

Surely, if the "Grothendieck group" of a semigroup means something, then then it is a group. The question is how to define it, how to compute it, and whether, if I start with a monoid, the Grothendieck group changes if I regard it instead as a semigroup.

Yaël Dillies (Apr 05 2023 at 07:11):

The paper I'm following defines localization (⊤ : subsemigroup α) and then claims it's a group without mentioning the possibility of it being empty.

Johan Commelin (Apr 05 2023 at 07:12):

Where α has an ambient structure of semigroup, or something stronger?

Yaël Dillies (Apr 05 2023 at 07:13):

comm_semigroup α is what the paper claims is sufficient (and I believe it, except for adding nonempty α)

Johan Commelin (Apr 05 2023 at 07:16):

Every map from an empty (comm)semigroup α to a group G factors uniquely via a group with one element. So do you really need to add that assumption?

Yaël Dillies (Apr 05 2023 at 07:18):

Am I right in saying that localization (⊤ : subsemigroup empty) is empty? If so, yes I do need that assumption to follow the paper's argument.

Yaël Dillies (Apr 05 2023 at 07:19):

I'm sure there's a separate argument that works for empty semigroups, just not the one that the paper is offering.

Reid Barton (Apr 05 2023 at 07:20):

I am not sure a priori that localization of semigroups makes sense at all.

Yaël Dillies (Apr 05 2023 at 07:21):

Read the paper :wink:

Reid Barton (Apr 05 2023 at 07:21):

Because "invertibility" of elements of a semigroup is not preserved by homomorphisms, like it is for monoids.

Johan Commelin (Apr 05 2023 at 07:21):

Yaël Dillies said:

Am I right in saying that localization (⊤ : subsemigroup empty) is empty? If so, yes I do need that assumption to follow the paper's argument.

That depends on what localization means. Despite suggestively writing it between backticks, I don't think Lean can answer that question in the current context.

Reid Barton (Apr 05 2023 at 07:22):

You are confusing the construction and the definition. I totally agree that the same construction used to define the Grothendieck group of a commutative monoid can also be applied to a commutative semigroup provided that the semigroup is nonempty.

Reid Barton (Apr 05 2023 at 07:26):

But I don't know what it means (if anything) to say that the result is the "localization of the semigroup" at all its elements.

Reid Barton (Apr 05 2023 at 07:28):

A thing you can definitely do is consider the universal abelian group with a map of semigroups from your original commutative semigroup A, and I believe it will be the thing in the paper if A is nonempty and the zero group if A is empty.

Yaël Dillies (Apr 05 2023 at 07:30):

Yeah that's probably the correct answer in general


Last updated: Dec 20 2023 at 11:08 UTC