Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit b29ab1b

Browse files
committed
feat(data/finsupp): add support_neg
1 parent a2d6148 commit b29ab1b

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

data/finsupp.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -239,6 +239,12 @@ rfl
239239
(g₁ - g₂) a = g₁ a - g₂ a :=
240240
rfl
241241

242+
@[simp] lemma support_neg [add_group β] {f : α →₀ β} : support (-f) = support f :=
243+
finset.subset.antisymm
244+
support_map_range
245+
(calc support f = support (- (- f)) : by simp
246+
... ⊆ support (- f) : support_map_range)
247+
242248
instance [add_comm_group β] : add_comm_group (α →₀ β) :=
243249
{ add_comm := add_comm, ..finsupp.add_group }
244250

0 commit comments

Comments
 (0)