Skip to content

Commit b6e8469

Browse files
feat: add mulTSupport_mul/tsupport_add (#9060)
From the hairer branch.
1 parent d61c95e commit b6e8469

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

Mathlib/Topology/Support.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -102,6 +102,13 @@ theorem tsupport_smul_subset_left {M α} [TopologicalSpace X] [Zero M] [Zero α]
102102
closure_mono <| support_smul_subset_left f g
103103
#align tsupport_smul_subset_left tsupport_smul_subset_left
104104

105+
@[to_additive]
106+
theorem mulTSupport_mul [TopologicalSpace X] [Monoid α] {f g : X → α} :
107+
(mulTSupport fun x ↦ f x * g x) ⊆ mulTSupport f ∪ mulTSupport g :=
108+
closure_minimal
109+
((mulSupport_mul f g).trans (union_subset_union (subset_mulTSupport _) (subset_mulTSupport _)))
110+
(isClosed_closure.union isClosed_closure)
111+
105112
section
106113

107114
variable [TopologicalSpace α] [TopologicalSpace α']

0 commit comments

Comments
 (0)