Zulip Chat Archive

Stream: Is there code for X?

Topic: mkq = 0 iff


Scott Morrison (Mar 09 2022 at 10:22):

import linear_algebra.quotient

lemma foo {R : Type*} [ring R] {M : Type*} [add_comm_group M] [module R M]
  (p : submodule R M) (x : M) : p.mkq x = 0  x  p :=
sorry

This seems like a core part of the API for submodule.mpq, but I can't seem to find it ....? Any pointers?

Riccardo Brasca (Mar 09 2022 at 10:24):

docs#submodule.ker_mkq?

Scott Morrison (Mar 09 2022 at 10:34):

I guess that is the pointless version. :-)

Scott Morrison (Mar 09 2022 at 10:35):

I will add this later.

Riccardo Brasca (Mar 09 2022 at 10:36):

Ah ops! docs#submodule.quotient.mk_eq_zero then, but it uses quotient.mk

Riccardo Brasca (Mar 09 2022 at 11:02):

But the two are defeq, indeed

lemma foo {R : Type*} [ring R] {M : Type*} [add_comm_group M] [module R M]
  (p : submodule R M) (x : M) : p.mkq x = 0  x  p :=
submodule.quotient.mk_eq_zero p

works.

Scott Morrison (Mar 09 2022 at 18:22):

Ah, I should have tried library_search!.

Scott Morrison (Mar 13 2022 at 08:13):

I added another copy of this lemma stated in terms of mkq so that simp can use it, in #12639.


Last updated: Dec 20 2023 at 11:08 UTC