-
Notifications
You must be signed in to change notification settings - Fork 298
feat(topology/algebra/infinite_sum): Extract none
from a sum over option
types
#19150
base: master
Are you sure you want to change the base?
Conversation
I think you want |
none
from a some over option
typesnone
from a sum over option
types
I also added versions for |
@@ -164,6 +164,11 @@ begin | |||
exact if_neg hb' | |||
end | |||
|
|||
lemma has_sum_singleton (f : β → α) (b : β) : has_sum (f ∘ coe : ({b} : set β) → α) (f b) := |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
Please add it for a [unique]
type, not just a singleton.
@@ -313,6 +318,16 @@ lemma has_sum.compl_add {s : set β} (ha : has_sum (f ∘ coe : sᶜ → α) a) | |||
has_sum f (a + b) := | |||
ha.add_is_compl is_compl_compl.symm hb | |||
|
|||
lemma has_sum.sum_t {f : β ⊕ γ → α} {a_inl a_inr : α} (h_inl : has_sum (f ∘ sum.inl) a_inl) |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
There are two ways to state this lemma: starting with β ⊕ γ → α
and starting with two functions and combining them using sum.elim
. Please add the second version too (the proof should be by application of this version). I'm not sure about the naming convention for this kind of lemmas. sum_dom
? I would ask on Zulip.
has_sum.add_is_compl (set.is_compl_range_inl_range_inr) | ||
(sum.inl_injective.has_sum_range_iff.2 h_inl) (sum.inr_injective.has_sum_range_iff.2 h_inr) | ||
|
||
lemma has_sum.option {f : option β → α} {a_some : α} (hf : has_sum (f ∘ option.some) a_some) : |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
Please make it protected
.
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
Also, please add summable
versions of your lemmas (with iff
versions whenever we can apply summable.comp_injective
).
This PR gives lemmas for separating a sum over
option α
into the value atnone
plus a sum overα