Zulip Chat Archive
Stream: Is there code for X?
Topic: Algebra map is injective
Thomas Browning (Jul 25 2021 at 19:50):
What's the best way to prove function.injective (algebra_map ℤ ℂ)
? Judging by some old code I had lying around, it seems like int.cast_injective
used to work, but now it looks like algebra_map ℤ ℂ
is not defeq to coe
.
Alex J. Best (Jul 25 2021 at 20:17):
import data.complex.basic
lemma hi : function.injective (algebra_map ℤ ℂ) := int.cast_injective
#print hi
works for me in the web editor
Eric Wieser (Jul 25 2021 at 20:46):
There are multiple non-defeq z-algebra instances
Eric Wieser (Jul 25 2021 at 20:46):
Which one you get depends on your imports along with other things
Eric Wieser (Jul 25 2021 at 20:47):
by convert int.cast_injective
should work
Eric Wieser (Jul 25 2021 at 20:49):
I think adding add_comm_monoid.of_nat
and add_comm_group.of_int
would fix this.
Eric Wieser (Jul 25 2021 at 21:00):
(this is in the future work section of my FMM 2021 paper)
Last updated: Dec 20 2023 at 11:08 UTC