Zulip Chat Archive
Stream: Is there code for X?
Topic: surjective Pi.evalMonoidHom
Jireh Loreaux (Oct 31 2023 at 15:59):
What's the right lemma that's supposed to prove this? Surely we have it.
theorem Pi.surjective_evalMonoidHom {I : Type*} (f : I → Type*) [(i : I) → MulOneClass (f i)]
(i : I) : Function.Surjective (evalMonoidHom f i) :=
fun g ↦ ⟨mulSingle i g, by simp⟩
Yaël Dillies (Oct 31 2023 at 16:25):
docs#Function.surjective_eval ?
Jireh Loreaux (Oct 31 2023 at 16:30):
Yaël search for the win. I was looking for Pi.surjective_eval
.
Last updated: Dec 20 2023 at 11:08 UTC