Zulip Chat Archive
Stream: mathlib4
Topic: Does the homogeneousSubmodule form a graded ring?
Pan Lin (Jul 14 2024 at 16:46):
The document says that:
instance MvPolynomial.IsHomogeneous.HomogeneousSubmodule.gcommSemiring{σ : Type u_1} {R : Type u_3} [CommSemiring R] :
SetLike.GradedMonoid (MvPolynomial.homogeneousSubmodule σ R)
The homogeneous submodules form a graded ring. This instance is used by
[DirectSum.commSemiring](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/DirectSum/Ring.html#DirectSum.commSemiring)
andDirectSum.algebra
.
But why there is no instance DirectSum.Decomposition (MvPolynomial.homogeneousSubmodule σ R)
to make the instance GradedRing (MvPolynomial.homogeneousSubmodule σ R)
?
Eric Wieser (Jul 14 2024 at 16:47):
(to write links with a code title, you want [`code`](link)
not `[code](link)`
)
Eric Wieser (Jul 14 2024 at 16:48):
(Or just remove the links, I don't think they're helping here)
Eric Wieser (Jul 14 2024 at 16:49):
(speculating: Ctrl+Shift+V lets you paste into zulip without keeping the unwanted formatting)
Riccardo Brasca (Jul 14 2024 at 17:03):
#14225 does it
Pan Lin (Jul 15 2024 at 09:00):
Riccardo Brasca 发言道:
#14225 does it
How can I use it?
Johan Commelin (Jul 15 2024 at 09:20):
That PR is waiting for its author to process some review comments. Hopefully it will be merged into mathlib soon.
Last updated: May 02 2025 at 03:31 UTC