Zulip Chat Archive
Stream: general
Topic: subalgebra.coe_top and friends
Scott Morrison (Apr 22 2021 at 11:37):
Currently src#subalgebra.coe_top reads
@[simp] theorem coe_top : (⊤ : subalgebra R A).to_submodule = ⊤ :=
submodule.ext $ λ x, iff_of_true mem_top trivial
It seems to me there's another theorem equally deserving that name, replacing to_submodule
with to_subsemiring
.
Similarly, coe_bot
is above the coercion to set
. This is all a bit confusing, and in any case incomplete.
Any suggestions about a good naming scheme for such lemmas? (@Eric Wieser?)
Eric Wieser (Apr 22 2021 at 11:40):
top_to_submodule
, to match docs#submodule.top_to_add_submonoid?
Eric Wieser (Apr 22 2021 at 11:40):
There's not a coe in that statement at all!
Eric Wieser (Apr 22 2021 at 11:41):
(docs#submodule.coe_top says ↑⊤ = set.univ
, which is what I'd expect it to say)
Last updated: Dec 20 2023 at 11:08 UTC