Zulip Chat Archive
Stream: Is there code for X?
Topic: x +ᵥ A = {x} + A
Mitchell Lee (Mar 27 2024 at 03:18):
Hello, is there any one-line proof of this in mathlib?
import Mathlib
open scoped Pointwise
example {M : Type} [Add M] (x : M) (A : Set M) : x +ᵥ A = {x} + A := by
sorry
Matt Diamond (Mar 27 2024 at 03:47):
idk if there's a lemma, but you can solve it with by rw [Set.singleton_add]; rfl
Mitchell Lee (Mar 27 2024 at 03:47):
Thanks
Yaël Dillies (Mar 27 2024 at 07:33):
Yes that's supposed to be docs#Set.singleton_add but it's currently misstated. I have been trying to fix it for more than a year :smiling_face_with_tear:
Last updated: May 02 2025 at 03:31 UTC