File tree Expand file tree Collapse file tree 1 file changed +9
-0
lines changed
Mathlib/Topology/Algebra/InfiniteSum Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Original file line number Diff line number Diff line change @@ -81,6 +81,15 @@ theorem tprod_le_tprod_of_inj {g : κ → α} (e : ι → κ) (he : Injective e)
81
81
hasProd_le_inj _ he hs h hf.hasProd hg.hasProd
82
82
#align tsum_le_tsum_of_inj tsum_le_tsum_of_inj
83
83
84
+ @[to_additive]
85
+ lemma tprod_subtype_le {κ γ : Type *} [OrderedCommGroup γ] [UniformSpace γ] [UniformGroup γ]
86
+ [OrderClosedTopology γ] [ CompleteSpace γ] (f : κ → γ) (β : Set κ) (h : ∀ a : κ, 1 ≤ f a)
87
+ (hf : Multipliable f) : (∏' (b : β), f b) ≤ (∏' (a : κ), f a) := by
88
+ apply tprod_le_tprod_of_inj _ (Subtype.coe_injective) (by simp only [Subtype.range_coe_subtype,
89
+ Set.setOf_mem_eq, h, implies_true]) (by simp only [le_refl,
90
+ Subtype.forall, implies_true]) (by apply hf.subtype)
91
+ apply hf
92
+
84
93
@[to_additive]
85
94
theorem prod_le_hasProd (s : Finset ι) (hs : ∀ i, i ∉ s → 1 ≤ f i) (hf : HasProd f a) :
86
95
∏ i ∈ s, f i ≤ a :=
You can’t perform that action at this time.
0 commit comments