Commit 2025-04-13 16:12 e8a574a8

View on Github →

chore(tprod): move tprod lemmas to protected namespace (#23959) As per zulip discussion, this PR renames lemmas of the form theorem tprod_foo {f : a -> b} (Multipliable f) : _ to protected theorem Multipliable.tprod_foo {f : a -> b} (Multipliable f) : _, and similar for tsum/Summable, usually via to_additive. This is so the name tprod_foo (and by extension tsum_foo) is freed up for planned versions of the lemmas in settings where multipliabilty/summability automatically holds (such as ENat and ENNReal for summability). We also deprecate all the old names.

Estimated changes

deleted theorem tprod_comm'
deleted theorem tprod_comm
deleted theorem tprod_prod'
deleted theorem tprod_prod
deleted theorem tprod_prod_uncurry
deleted theorem tprod_sigma'
deleted theorem tprod_sigma
deleted theorem tprod_sum
deleted theorem abs_tprod
deleted theorem le_tprod'
deleted theorem le_tprod
deleted theorem one_lt_tprod
deleted theorem prod_le_tprod
deleted theorem tprod_eq_one_iff
deleted theorem tprod_le_of_prod_le
deleted theorem tprod_le_of_prod_range_le
deleted theorem tprod_le_tprod
deleted theorem tprod_le_tprod_of_inj
deleted theorem tprod_lt_tprod
deleted theorem tprod_mono
deleted theorem tprod_ne_one_iff
deleted theorem tprod_strict_mono
deleted theorem tprod_subtype_le