Zulip Chat Archive

Stream: Is there code for X?

Topic: ring homomorphism commuting with direct sum inclusion


Jujian Zhang (Oct 25 2021 at 17:10):

f is a homomorphism between graded rings, is there a short proof for f commuting with of where of B i is the inclusion from BiiBiB_i \to \oplus_i B_i and similar for of A i, i.e. the following:

example {ι : Type*} [add_comm_monoid ι] (A B : ι  Type*) [Π (i : ι), add_comm_monoid (A i)]
  [Π (i : ι), add_comm_monoid (B i)] [gcomm_semiring A] [gcomm_semiring B]
  (f : ( i, A i) →+* ( i, B i)) (i : ι) (x :  i, A i) :
  f (of A i (x i)) = of B i ((f x) i) := sorry

Johan Commelin (Oct 25 2021 at 17:12):

@Jujian Zhang that's not true in general right? A hom of graded rings is a ring hom + a proof that it preserves the grading.

Johan Commelin (Oct 25 2021 at 17:15):

Also, not every graded ring in mathlib will be defeq to ⨁ i, A i, right? Something like mv_polynomial isn't of that shape. So I think a morphism of graded rings should take that into account.

Kevin Buzzard (Oct 25 2021 at 17:15):

I guess a counterexample would be the map on polynomial rings k[X]k[X]k[X]\to k[X] sending XX to X2X^2.


Last updated: Dec 20 2023 at 11:08 UTC