Zulip Chat Archive
Stream: toric
Topic: Refactoring torus definition
Michał Mrugała (Feb 25 2025 at 14:21):
I think it's a good idea to adapt our definition of a torus with Andrew's work on group schemes. We essentially only need to lift his results to the over category.
Yaël Dillies (Feb 25 2025 at 14:22):
Where are Andrew's group schemes?
Michał Mrugała (Feb 25 2025 at 14:23):
GroupScheme.lean (currently not in mathlib)
Michał Mrugała (Feb 25 2025 at 14:26):
As a subtask, it would be good to replace the Mathlib import by smaller imports in that file.
Andrew Yang (Feb 26 2025 at 17:00):
We are lacking a fair bit of rudimentary API on group-objects though. #22168 would be a start.
But someone need to generalize the docs#CategoryTheory.Mon_ClassOfRepresentableBy to CommGrp_Class
(where CommGrp_Class
doesn't even exist yet)
Would be nice if developing them are a part of this project.
Michał Mrugała (Feb 26 2025 at 17:03):
I'd be happy to work on this after I manage to formalize the defintion of toric ideals. We will need basic results about tori for our first bigger objective, so developing the API is probably necessary.
Andrew Yang (Feb 26 2025 at 17:14):
Also one would need to change docs#FreeAbelianGroup to Finsupp so that the definition is defeq to MvLaurentPolynomial
Andrew Yang (Feb 26 2025 at 17:15):
(or just change docs#AddCommGrp.free if people are lazy like me)
Yaël Dillies (Apr 03 2025 at 15:33):
I am trying to understand what SplitTorus
is defined as, informally. Am I right in saying it's something like R ⊗ ℤ[ℤⁿ]
?
Michał Mrugała (Apr 03 2025 at 15:42):
That’s one way to view it yeah
Yaël Dillies (Apr 03 2025 at 15:43):
But is it defined like this?
Michał Mrugała (Apr 03 2025 at 15:47):
It’s defined as a pullback which will be isomorphic to the spectrum of the ring you wrote down
Michał Mrugała (Apr 03 2025 at 15:47):
The isomorphism should be in mathlib (if it’s not then we really ought to prove it)
Kevin Buzzard (Apr 03 2025 at 16:48):
A split torus over should really be Spec(R[G]) where G is a group isomorphic to (but without a fixed isomorphism) (or just R[G] if you're happy with the Hopf algebra rather than the affine R-group-scheme).
Yaël Dillies (Apr 03 2025 at 17:01):
But what about a split torus over an arbitrary scheme? This is what Andrew defined
Kevin Buzzard (Apr 03 2025 at 17:09):
Well that's relative Spec of O_X[G] where G is a group isomorphic to Z^n. Here O_X is the structure sheaf of the scheme (so O_X is to X as R is to Spec(R)) and given a sheaf of algebras for the sheaf of rings you can take relative spec and get a scheme mapping to X with affine fibres.
Sophie Morel (Apr 04 2025 at 09:21):
Do we have relative Spec
s already?
Yaël Dillies (Apr 04 2025 at 09:24):
Do you mean something like algSpec
?
Michał Mrugała (Apr 04 2025 at 09:26):
That’s not it, this is what Kevin and Sophie are talking about: https://stacks.math.columbia.edu/tag/01LQ
Sophie Morel (Apr 04 2025 at 09:30):
And I realize that my question was naive, I don't think the theory of quasi-coherent sheaves is developed enough for that.
Kevin Buzzard (Apr 04 2025 at 09:36):
Oh I guess another definition of "split torus over S" is "S-group-scheme isomorphic to S x_Z Spec(Z[Z^n]) for some natural"
Andrew Yang (Apr 04 2025 at 09:54):
@Christian Merten has some code on relative specs IIRC.
Andrew Yang (Apr 04 2025 at 09:55):
Kevin Buzzard said:
S-group-scheme isomorphic to S x_Z Spec(Z[Z^n]) for some natural
Yeah that is the proposed definition.
Christian Merten (Apr 04 2025 at 11:54):
Andrew Yang said:
Christian Merten has some code on relative specs IIRC.
Not really anything usable, I gave up because, as Sophie said, it seemed pointless as long as we don't have more on quasi-coherent sheaves.
Last updated: May 02 2025 at 03:31 UTC