formal
stringlengths 41
427k
| informal
stringclasses 1
value |
---|---|
intervalIntegral.norm_intervalIntegral_eq ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ✝ : Measure ℝ f : ℝ → E a b : ℝ μ : Measure ℝ ⊢ ‖∫ (x : ℝ) in a..b, f x ∂μ‖ = ‖∫ (x : ℝ) in Ι a b, f x ∂μ‖ ** simp_rw [intervalIntegral_eq_integral_uIoc, norm_smul] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ✝ : Measure ℝ f : ℝ → E a b : ℝ μ : Measure ℝ ⊢ ‖if a ≤ b then 1 else -1‖ * ‖∫ (x : ℝ) in Ι a b, f x ∂μ‖ = ‖∫ (x : ℝ) in Ι a b, f x ∂μ‖ ** split_ifs <;> simp only [norm_neg, norm_one, one_mul] ** Qed
| |
intervalIntegral.integral_cases ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ : Measure ℝ f : ℝ → E a b : ℝ ⊢ ∫ (x : ℝ) in a..b, f x ∂μ ∈ {∫ (x : ℝ) in Ι a b, f x ∂μ, -∫ (x : ℝ) in Ι a b, f x ∂μ} ** rw [intervalIntegral_eq_integral_uIoc] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ : Measure ℝ f : ℝ → E a b : ℝ ⊢ (if a ≤ b then 1 else -1) • ∫ (x : ℝ) in Ι a b, f x ∂μ ∈ {∫ (x : ℝ) in Ι a b, f x ∂μ, -∫ (x : ℝ) in Ι a b, f x ∂μ} ** split_ifs <;> simp ** Qed
| |
intervalIntegral.integral_undef ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ h : ¬IntervalIntegrable f μ a b ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ** rw [intervalIntegrable_iff] at h ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ h : ¬IntegrableOn f (Ι a b) ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ** rw [intervalIntegral_eq_integral_uIoc, integral_undef h, smul_zero] ** Qed
| |
intervalIntegral.integral_non_aestronglyMeasurable ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ hf : ¬AEStronglyMeasurable f (Measure.restrict μ (Ι a b)) ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ** rw [intervalIntegral_eq_integral_uIoc, integral_non_aestronglyMeasurable hf, smul_zero] ** Qed
| |
intervalIntegral.norm_integral_min_max ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f✝ g : ℝ → E μ : Measure ℝ f : ℝ → E ⊢ ‖∫ (x : ℝ) in min a b..max a b, f x ∂μ‖ = ‖∫ (x : ℝ) in a..b, f x ∂μ‖ ** cases le_total a b <;> simp [*, integral_symm a b] ** Qed
| |
intervalIntegral.norm_integral_le_abs_integral_norm ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ ⊢ ‖∫ (x : ℝ) in a..b, f x ∂μ‖ ≤ |∫ (x : ℝ) in a..b, ‖f x‖ ∂μ| ** simp only [← Real.norm_eq_abs, norm_integral_eq_norm_integral_Ioc] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ ⊢ ‖∫ (x : ℝ) in Ι a b, f x ∂μ‖ ≤ ‖∫ (x : ℝ) in Ι a b, ‖f x‖ ∂μ‖ ** exact le_trans (norm_integral_le_integral_norm _) (le_abs_self _) ** Qed
| |
intervalIntegral.norm_integral_le_integral_norm ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ h : a ≤ b ⊢ ∫ (x : ℝ) in Ι a b, ‖f x‖ ∂μ = ∫ (x : ℝ) in a..b, ‖f x‖ ∂μ ** rw [uIoc_of_le h, integral_of_le h] ** Qed
| |
intervalIntegral.norm_integral_le_of_norm_le_const_ae ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ : Measure ℝ a b C : ℝ f : ℝ → E h : ∀ᵐ (x : ℝ), x ∈ Ι a b → ‖f x‖ ≤ C ⊢ ‖∫ (x : ℝ) in a..b, f x‖ ≤ C * |b - a| ** rw [norm_integral_eq_norm_integral_Ioc] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ : Measure ℝ a b C : ℝ f : ℝ → E h : ∀ᵐ (x : ℝ), x ∈ Ι a b → ‖f x‖ ≤ C ⊢ ‖∫ (x : ℝ) in Ι a b, f x‖ ≤ C * |b - a| ** convert norm_set_integral_le_of_norm_le_const_ae'' _ measurableSet_Ioc h using 1 ** case h.e'_4 ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ : Measure ℝ a b C : ℝ f : ℝ → E h : ∀ᵐ (x : ℝ), x ∈ Ι a b → ‖f x‖ ≤ C ⊢ C * |b - a| = C * ENNReal.toReal (↑↑volume (Ioc (min a b) (max a b))) ** rw [Real.volume_Ioc, max_sub_min_eq_abs, ENNReal.toReal_ofReal (abs_nonneg _)] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ : ℝ f✝ g : ℝ → E μ : Measure ℝ a b C : ℝ f : ℝ → E h : ∀ᵐ (x : ℝ), x ∈ Ι a b → ‖f x‖ ≤ C ⊢ ↑↑volume (Ioc (min a b) (max a b)) < ⊤ ** simp only [Real.volume_Ioc, ENNReal.ofReal_lt_top] ** Qed
| |
intervalIntegral.integral_add ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b ⊢ ∫ (x : ℝ) in a..b, f x + g x ∂μ = ∫ (x : ℝ) in a..b, f x ∂μ + ∫ (x : ℝ) in a..b, g x ∂μ ** simp only [intervalIntegral_eq_integral_uIoc, integral_add hf.def hg.def, smul_add] ** Qed
| |
intervalIntegral.integral_neg ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ ⊢ ∫ (x : ℝ) in a..b, -f x ∂μ = -∫ (x : ℝ) in a..b, f x ∂μ ** simp only [intervalIntegral, integral_neg] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ ⊢ -∫ (a : ℝ) in Ioc a b, f a ∂μ - -∫ (a : ℝ) in Ioc b a, f a ∂μ = -(∫ (a : ℝ) in Ioc a b, f a ∂μ - ∫ (a : ℝ) in Ioc b a, f a ∂μ) ** abel ** Qed
| |
intervalIntegral.integral_sub ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b ⊢ ∫ (x : ℝ) in a..b, f x - g x ∂μ = ∫ (x : ℝ) in a..b, f x ∂μ - ∫ (x : ℝ) in a..b, g x ∂μ ** simpa only [sub_eq_add_neg] using (integral_add hf hg.neg).trans (congr_arg _ integral_neg) ** Qed
| |
intervalIntegral.integral_smul ** ι : Type u_1 𝕜✝ : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝⁵ : NormedAddCommGroup E inst✝⁴ : CompleteSpace E inst✝³ : NormedSpace ℝ E a b : ℝ f✝ g : ℝ → E μ : Measure ℝ 𝕜 : Type u_6 inst✝² : NontriviallyNormedField 𝕜 inst✝¹ : NormedSpace 𝕜 E inst✝ : SMulCommClass ℝ 𝕜 E r : 𝕜 f : ℝ → E ⊢ ∫ (x : ℝ) in a..b, r • f x ∂μ = r • ∫ (x : ℝ) in a..b, f x ∂μ ** simp only [intervalIntegral, integral_smul, smul_sub] ** Qed
| |
intervalIntegral.integral_smul_const ** ι : Type u_1 𝕜✝ : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝⁴ : NormedAddCommGroup E inst✝³ : CompleteSpace E inst✝² : NormedSpace ℝ E a b : ℝ f✝ g : ℝ → E μ : Measure ℝ 𝕜 : Type u_6 inst✝¹ : IsROrC 𝕜 inst✝ : NormedSpace 𝕜 E f : ℝ → 𝕜 c : E ⊢ ∫ (x : ℝ) in a..b, f x • c ∂μ = (∫ (x : ℝ) in a..b, f x ∂μ) • c ** simp only [intervalIntegral_eq_integral_uIoc, integral_smul_const, smul_assoc] ** Qed
| |
intervalIntegral.integral_mul_const ** ι : Type u_1 𝕜✝ : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b : ℝ f✝ g : ℝ → E μ : Measure ℝ 𝕜 : Type u_6 inst✝ : IsROrC 𝕜 r : 𝕜 f : ℝ → 𝕜 ⊢ ∫ (x : ℝ) in a..b, f x * r ∂μ = (∫ (x : ℝ) in a..b, f x ∂μ) * r ** simpa only [mul_comm r] using integral_const_mul r f ** Qed
| |
intervalIntegral.integral_const' ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ c : E ⊢ ∫ (x : ℝ) in a..b, c ∂μ = (ENNReal.toReal (↑↑μ (Ioc a b)) - ENNReal.toReal (↑↑μ (Ioc b a))) • c ** simp only [intervalIntegral, set_integral_const, sub_smul] ** Qed
| |
intervalIntegral.integral_smul_measure ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b : ℝ f g : ℝ → E μ : Measure ℝ c : ℝ≥0∞ ⊢ ∫ (x : ℝ) in a..b, f x ∂c • μ = ENNReal.toReal c • ∫ (x : ℝ) in a..b, f x ∂μ ** simp only [intervalIntegral, Measure.restrict_smul, integral_smul_measure, smul_sub] ** Qed
| |
ContinuousLinearMap.intervalIntegral_apply ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝⁶ : NormedAddCommGroup E inst✝⁵ : CompleteSpace E inst✝⁴ : NormedSpace ℝ E a✝ b✝ : ℝ μ : Measure ℝ f : ℝ → E inst✝³ : IsROrC 𝕜 inst✝² : NormedSpace 𝕜 E inst✝¹ : NormedAddCommGroup F inst✝ : NormedSpace 𝕜 F a b : ℝ φ : ℝ → F →L[𝕜] E hφ : IntervalIntegrable φ μ a b v : F ⊢ ↑(∫ (x : ℝ) in a..b, φ x ∂μ) v = ∫ (x : ℝ) in a..b, ↑(φ x) v ∂μ ** simp_rw [intervalIntegral_eq_integral_uIoc, ← integral_apply hφ.def v, coe_smul', Pi.smul_apply] ** Qed
| |
ContinuousLinearMap.intervalIntegral_comp_comm ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝⁸ : NormedAddCommGroup E inst✝⁷ : CompleteSpace E inst✝⁶ : NormedSpace ℝ E a b : ℝ μ : Measure ℝ f : ℝ → E inst✝⁵ : IsROrC 𝕜 inst✝⁴ : NormedSpace 𝕜 E inst✝³ : NormedAddCommGroup F inst✝² : NormedSpace 𝕜 F inst✝¹ : NormedSpace ℝ F inst✝ : CompleteSpace F L : E →L[𝕜] F hf : IntervalIntegrable f μ a b ⊢ ∫ (x : ℝ) in a..b, ↑L (f x) ∂μ = ↑L (∫ (x : ℝ) in a..b, f x ∂μ) ** simp_rw [intervalIntegral, L.integral_comp_comm hf.1, L.integral_comp_comm hf.2, L.map_sub] ** Qed
| |
intervalIntegral.smul_integral_comp_mul_right ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d : ℝ f : ℝ → E c : ℝ ⊢ c • ∫ (x : ℝ) in a..b, f (x * c) = ∫ (x : ℝ) in a * c..b * c, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_mul_right] ** Qed
| |
intervalIntegral.integral_comp_mul_left ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f : ℝ → E hc : c ≠ 0 ⊢ ∫ (x : ℝ) in a..b, f (c * x) = c⁻¹ • ∫ (x : ℝ) in c * a..c * b, f x ** simpa only [mul_comm c] using integral_comp_mul_right f hc ** Qed
| |
intervalIntegral.smul_integral_comp_mul_left ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d : ℝ f : ℝ → E c : ℝ ⊢ c • ∫ (x : ℝ) in a..b, f (c * x) = ∫ (x : ℝ) in c * a..c * b, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_mul_left] ** Qed
| |
intervalIntegral.integral_comp_div ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f : ℝ → E hc : c ≠ 0 ⊢ ∫ (x : ℝ) in a..b, f (x / c) = c • ∫ (x : ℝ) in a / c..b / c, f x ** simpa only [inv_inv] using integral_comp_mul_right f (inv_ne_zero hc) ** Qed
| |
intervalIntegral.inv_smul_integral_comp_div ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d : ℝ f : ℝ → E c : ℝ ⊢ c⁻¹ • ∫ (x : ℝ) in a..b, f (x / c) = ∫ (x : ℝ) in a / c..b / c, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_div] ** Qed
| |
intervalIntegral.integral_comp_add_right ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A✝ : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E d : ℝ A : MeasurableEmbedding fun x => x + d ⊢ ∫ (x : ℝ) in a..b, f (x + d) = ∫ (x : ℝ) in a + d..b + d, f x ∂Measure.map (fun x => x + d) volume ** simp [intervalIntegral, A.set_integral_map] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A✝ : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E d : ℝ A : MeasurableEmbedding fun x => x + d ⊢ ∫ (x : ℝ) in a + d..b + d, f x ∂Measure.map (fun x => x + d) volume = ∫ (x : ℝ) in a + d..b + d, f x ** rw [map_add_right_eq_self] ** Qed
| |
intervalIntegral.integral_comp_add_left ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (d + x) = ∫ (x : ℝ) in d + a..d + b, f x ** simpa only [add_comm d] using integral_comp_add_right f d ** Qed
| |
intervalIntegral.integral_comp_mul_add ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (c * x + d) = c⁻¹ • ∫ (x : ℝ) in c * a + d..c * b + d, f x ** rw [← integral_comp_add_right, ← integral_comp_mul_left _ hc] ** Qed
| |
intervalIntegral.smul_integral_comp_mul_add ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d✝ : ℝ f : ℝ → E c d : ℝ ⊢ c • ∫ (x : ℝ) in a..b, f (c * x + d) = ∫ (x : ℝ) in c * a + d..c * b + d, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_mul_add] ** Qed
| |
intervalIntegral.smul_integral_comp_add_mul ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d✝ : ℝ f : ℝ → E c d : ℝ ⊢ c • ∫ (x : ℝ) in a..b, f (d + c * x) = ∫ (x : ℝ) in d + c * a..d + c * b, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_add_mul] ** Qed
| |
intervalIntegral.integral_comp_div_add ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (x / c + d) = c • ∫ (x : ℝ) in a / c + d..b / c + d, f x ** simpa only [div_eq_inv_mul, inv_inv] using integral_comp_mul_add f (inv_ne_zero hc) d ** Qed
| |
intervalIntegral.integral_comp_add_div ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (d + x / c) = c • ∫ (x : ℝ) in d + a / c..d + b / c, f x ** simpa only [div_eq_inv_mul, inv_inv] using integral_comp_add_mul f (inv_ne_zero hc) d ** Qed
| |
intervalIntegral.integral_comp_mul_sub ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (c * x - d) = c⁻¹ • ∫ (x : ℝ) in c * a - d..c * b - d, f x ** simpa only [sub_eq_add_neg] using integral_comp_mul_add f hc (-d) ** Qed
| |
intervalIntegral.smul_integral_comp_mul_sub ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d✝ : ℝ f : ℝ → E c d : ℝ ⊢ c • ∫ (x : ℝ) in a..b, f (c * x - d) = ∫ (x : ℝ) in c * a - d..c * b - d, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_mul_sub] ** Qed
| |
intervalIntegral.integral_comp_sub_mul ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (d - c * x) = c⁻¹ • ∫ (x : ℝ) in d - c * b..d - c * a, f x ** simp only [sub_eq_add_neg, neg_mul_eq_neg_mul] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (d + -c * x) = c⁻¹ • ∫ (x : ℝ) in d + -c * b..d + -c * a, f x ** rw [integral_comp_add_mul f (neg_ne_zero.mpr hc) d, integral_symm] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ (-c)⁻¹ • -∫ (x : ℝ) in d + -c * b..d + -c * a, f x = c⁻¹ • ∫ (x : ℝ) in d + -c * b..d + -c * a, f x ** simp only [inv_neg, smul_neg, neg_neg, neg_smul] ** Qed
| |
intervalIntegral.smul_integral_comp_sub_mul ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c✝ d✝ : ℝ f : ℝ → E c d : ℝ ⊢ c • ∫ (x : ℝ) in a..b, f (d - c * x) = ∫ (x : ℝ) in d - c * b..d - c * a, f x ** by_cases hc : c = 0 <;> simp [hc, integral_comp_sub_mul] ** Qed
| |
intervalIntegral.integral_comp_div_sub ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (x / c - d) = c • ∫ (x : ℝ) in a / c - d..b / c - d, f x ** simpa only [div_eq_inv_mul, inv_inv] using integral_comp_mul_sub f (inv_ne_zero hc) d ** Qed
| |
intervalIntegral.integral_comp_sub_div ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E hc : c ≠ 0 d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (d - x / c) = c • ∫ (x : ℝ) in d - b / c..d - a / c, f x ** simpa only [div_eq_inv_mul, inv_inv] using integral_comp_sub_mul f (inv_ne_zero hc) d ** Qed
| |
intervalIntegral.integral_comp_sub_right ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (x - d) = ∫ (x : ℝ) in a - d..b - d, f x ** simpa only [sub_eq_add_neg] using integral_comp_add_right f (-d) ** Qed
| |
intervalIntegral.integral_comp_sub_left ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d✝ : ℝ f : ℝ → E d : ℝ ⊢ ∫ (x : ℝ) in a..b, f (d - x) = ∫ (x : ℝ) in d - b..d - a, f x ** simpa only [one_mul, one_smul, inv_one] using integral_comp_sub_mul f one_ne_zero d ** Qed
| |
intervalIntegral.integral_comp_neg ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f : ℝ → E ⊢ ∫ (x : ℝ) in a..b, f (-x) = ∫ (x : ℝ) in -b..-a, f x ** simpa only [zero_sub] using integral_comp_sub_left f 0 ** Qed
| |
intervalIntegral.integral_congr ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ c d : ℝ f g : ℝ → E μ : Measure ℝ a b : ℝ h : EqOn f g [[a, b]] ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = ∫ (x : ℝ) in a..b, g x ∂μ ** cases' le_total a b with hab hab <;>
simpa [hab, integral_of_le, integral_of_ge] using
set_integral_congr measurableSet_Ioc (h.mono Ioc_subset_Icc_self) ** Qed
| |
intervalIntegral.sum_integral_adjacent_intervals_Ico ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n hint : ∀ (k : ℕ), k ∈ Ico m n → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ ∑ k in Finset.Ico m n, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a n, f x ∂μ ** revert hint ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n ⊢ (∀ (k : ℕ), k ∈ Ico m n → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m n, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a n, f x ∂μ ** refine' Nat.le_induction _ _ n hmn ** case refine'_1 ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n ⊢ (∀ (k : ℕ), k ∈ Ico m m → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m m, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a m, f x ∂μ ** simp ** case refine'_2 ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n ⊢ ∀ (n : ℕ), m ≤ n → ((∀ (k : ℕ), k ∈ Ico m n → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m n, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a n, f x ∂μ) → (∀ (k : ℕ), k ∈ Ico m (n + 1) → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m (n + 1), ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a (n + 1), f x ∂μ ** intro p hmp IH h ** case refine'_2 ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ ∑ k in Finset.Ico m (p + 1), ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a (p + 1), f x ∂μ ** rw [Finset.sum_Ico_succ_top hmp, IH, integral_add_adjacent_intervals] ** case refine'_2.hab ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ IntervalIntegrable (fun x => f x) μ (a m) (a p) ** refine IntervalIntegrable.trans_iterate_Ico hmp fun k hk => h k ?_ ** case refine'_2.hab ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) k : ℕ hk : k ∈ Ico m p ⊢ k ∈ Ico m (p + 1) ** exact (Ico_subset_Ico le_rfl (Nat.le_succ _)) hk ** case refine'_2.hbc ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ IntervalIntegrable (fun x => f x) μ (a p) (a (p + 1)) ** apply h ** case refine'_2.hbc.a ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ p ∈ Ico m (p + 1) ** simp [hmp] ** case refine'_2 ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ ∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1)) ** intro k hk ** case refine'_2 ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ m n : ℕ hmn : m ≤ n p : ℕ hmp : m ≤ p IH : (∀ (k : ℕ), k ∈ Ico m p → IntervalIntegrable f μ (a k) (a (k + 1))) → ∑ k in Finset.Ico m p, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a m..a p, f x ∂μ h : ∀ (k : ℕ), k ∈ Ico m (p + 1) → IntervalIntegrable f μ (a k) (a (k + 1)) k : ℕ hk : k ∈ Ico m p ⊢ IntervalIntegrable f μ (a k) (a (k + 1)) ** exact h _ (Ico_subset_Ico_right p.le_succ hk) ** Qed
| |
intervalIntegral.sum_integral_adjacent_intervals ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ n : ℕ hint : ∀ (k : ℕ), k < n → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ ∑ k in Finset.range n, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a 0 ..a n, f x ∂μ ** rw [← Nat.Ico_zero_eq_range] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b c d : ℝ f g : ℝ → E μ : Measure ℝ a : ℕ → ℝ n : ℕ hint : ∀ (k : ℕ), k < n → IntervalIntegrable f μ (a k) (a (k + 1)) ⊢ ∑ k in Finset.Ico 0 n, ∫ (x : ℝ) in a k..a (k + 1), f x ∂μ = ∫ (x : ℝ) in a 0 ..a n, f x ∂μ ** exact sum_integral_adjacent_intervals_Ico (zero_le n) fun k hk => hint k hk.2 ** Qed
| |
intervalIntegral.integral_interval_add_interval_comm ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ hab : IntervalIntegrable f μ a b hcd : IntervalIntegrable f μ c d hac : IntervalIntegrable f μ a c ⊢ ∫ (x : ℝ) in a..b, f x ∂μ + ∫ (x : ℝ) in c..d, f x ∂μ = ∫ (x : ℝ) in a..d, f x ∂μ + ∫ (x : ℝ) in c..b, f x ∂μ ** rw [← integral_add_adjacent_intervals hac hcd, add_assoc, add_left_comm,
integral_add_adjacent_intervals hac (hac.symm.trans hab), add_comm] ** Qed
| |
intervalIntegral.integral_eq_integral_of_support_subset ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ c d : ℝ f g : ℝ → E μ : Measure ℝ a b : ℝ h : support f ⊆ Ioc a b ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = ∫ (x : ℝ), f x ∂μ ** cases' le_total a b with hab hab ** case inl ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ c d : ℝ f g : ℝ → E μ : Measure ℝ a b : ℝ h : support f ⊆ Ioc a b hab : a ≤ b ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = ∫ (x : ℝ), f x ∂μ ** rw [integral_of_le hab, ← integral_indicator measurableSet_Ioc, indicator_eq_self.2 h] ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ c d : ℝ f g : ℝ → E μ : Measure ℝ a b : ℝ h : support f ⊆ Ioc a b hab : b ≤ a ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = ∫ (x : ℝ), f x ∂μ ** rw [Ioc_eq_empty hab.not_lt, subset_empty_iff, support_eq_empty_iff] at h ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a✝ b✝ c d : ℝ f g : ℝ → E μ : Measure ℝ a b : ℝ h : f = 0 hab : b ≤ a ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = ∫ (x : ℝ), f x ∂μ ** simp [h] ** Qed
| |
intervalIntegral.integral_congr_ae' ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ h : ∀ᵐ (x : ℝ) ∂μ, x ∈ Ioc a b → f x = g x h' : ∀ᵐ (x : ℝ) ∂μ, x ∈ Ioc b a → f x = g x ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = ∫ (x : ℝ) in a..b, g x ∂μ ** simp only [intervalIntegral, set_integral_congr_ae measurableSet_Ioc h,
set_integral_congr_ae measurableSet_Ioc h'] ** Qed
| |
intervalIntegral.integral_indicator ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ a₁ a₂ a₃ : ℝ h : a₂ ∈ Icc a₁ a₃ ⊢ ∫ (x : ℝ) in a₁..a₃, indicator {x | x ≤ a₂} f x ∂μ = ∫ (x : ℝ) in a₁..a₂, f x ∂μ ** have : {x | x ≤ a₂} ∩ Ioc a₁ a₃ = Ioc a₁ a₂ := Iic_inter_Ioc_of_le h.2 ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ a₁ a₂ a₃ : ℝ h : a₂ ∈ Icc a₁ a₃ this : {x | x ≤ a₂} ∩ Ioc a₁ a₃ = Ioc a₁ a₂ ⊢ ∫ (x : ℝ) in a₁..a₃, indicator {x | x ≤ a₂} f x ∂μ = ∫ (x : ℝ) in a₁..a₂, f x ∂μ ** rw [integral_of_le h.1, integral_of_le (h.1.trans h.2), integral_indicator,
Measure.restrict_restrict, this] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ a₁ a₂ a₃ : ℝ h : a₂ ∈ Icc a₁ a₃ this : {x | x ≤ a₂} ∩ Ioc a₁ a₃ = Ioc a₁ a₂ ⊢ MeasurableSet {x | x ≤ a₂} ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ a₁ a₂ a₃ : ℝ h : a₂ ∈ Icc a₁ a₃ this : {x | x ≤ a₂} ∩ Ioc a₁ a₃ = Ioc a₁ a₂ ⊢ MeasurableSet {x | x ≤ a₂} ** exact measurableSet_Iic ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ a₁ a₂ a₃ : ℝ h : a₂ ∈ Icc a₁ a₃ this : {x | x ≤ a₂} ∩ Ioc a₁ a₃ = Ioc a₁ a₂ ⊢ MeasurableSet {x | x ≤ a₂} ** all_goals apply measurableSet_Iic ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ a₁ a₂ a₃ : ℝ h : a₂ ∈ Icc a₁ a₃ this : {x | x ≤ a₂} ∩ Ioc a₁ a₃ = Ioc a₁ a₂ ⊢ MeasurableSet {x | x ≤ a₂} ** apply measurableSet_Iic ** Qed
| |
intervalIntegral.tendsto_integral_filter_of_dominated_convergence ** ι✝ : Type u_1 𝕜 : Type u_2 E : Type u_3 F✝ : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ ι : Type u_6 l : Filter ι inst✝ : IsCountablyGenerated l F : ι → ℝ → E bound : ℝ → ℝ hF_meas : ∀ᶠ (n : ι) in l, AEStronglyMeasurable (F n) (Measure.restrict μ (Ι a b)) h_bound : ∀ᶠ (n : ι) in l, ∀ᵐ (x : ℝ) ∂μ, x ∈ Ι a b → ‖F n x‖ ≤ bound x bound_integrable : IntervalIntegrable bound μ a b h_lim : ∀ᵐ (x : ℝ) ∂μ, x ∈ Ι a b → Tendsto (fun n => F n x) l (𝓝 (f x)) ⊢ Tendsto (fun n => ∫ (x : ℝ) in a..b, F n x ∂μ) l (𝓝 (∫ (x : ℝ) in a..b, f x ∂μ)) ** simp only [intervalIntegrable_iff, intervalIntegral_eq_integral_uIoc,
← ae_restrict_iff' (α := ℝ) (μ := μ) measurableSet_uIoc] at * ** ι✝ : Type u_1 𝕜 : Type u_2 E : Type u_3 F✝ : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ ι : Type u_6 l : Filter ι inst✝ : IsCountablyGenerated l F : ι → ℝ → E bound : ℝ → ℝ hF_meas : ∀ᶠ (n : ι) in l, AEStronglyMeasurable (F n) (Measure.restrict μ (Ι a b)) h_bound : ∀ᶠ (n : ι) in l, ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ι a b), ‖F n x‖ ≤ bound x bound_integrable : IntegrableOn bound (Ι a b) h_lim : ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ι a b), Tendsto (fun n => F n x) l (𝓝 (f x)) ⊢ Tendsto (fun n => (if a ≤ b then 1 else -1) • ∫ (x : ℝ) in Ι a b, F n x ∂μ) l (𝓝 ((if a ≤ b then 1 else -1) • ∫ (x : ℝ) in Ι a b, f x ∂μ)) ** exact tendsto_const_nhds.smul <|
tendsto_integral_filter_of_dominated_convergence bound hF_meas h_bound bound_integrable h_lim ** Qed
| |
intervalIntegral.hasSum_integral_of_dominated_convergence ** ι✝ : Type u_1 𝕜 : Type u_2 E : Type u_3 F✝ : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ ι : Type u_6 inst✝ : Countable ι F : ι → ℝ → E bound : ι → ℝ → ℝ hF_meas : ∀ (n : ι), AEStronglyMeasurable (F n) (Measure.restrict μ (Ι a b)) h_bound : ∀ (n : ι), ∀ᵐ (t : ℝ) ∂μ, t ∈ Ι a b → ‖F n t‖ ≤ bound n t bound_summable : ∀ᵐ (t : ℝ) ∂μ, t ∈ Ι a b → Summable fun n => bound n t bound_integrable : IntervalIntegrable (fun t => ∑' (n : ι), bound n t) μ a b h_lim : ∀ᵐ (t : ℝ) ∂μ, t ∈ Ι a b → HasSum (fun n => F n t) (f t) ⊢ HasSum (fun n => ∫ (t : ℝ) in a..b, F n t ∂μ) (∫ (t : ℝ) in a..b, f t ∂μ) ** simp only [intervalIntegrable_iff, intervalIntegral_eq_integral_uIoc, ←
ae_restrict_iff' (α := ℝ) (μ := μ) measurableSet_uIoc] at * ** ι✝ : Type u_1 𝕜 : Type u_2 E : Type u_3 F✝ : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b c d : ℝ f g : ℝ → E μ : Measure ℝ ι : Type u_6 inst✝ : Countable ι F : ι → ℝ → E bound : ι → ℝ → ℝ hF_meas : ∀ (n : ι), AEStronglyMeasurable (F n) (Measure.restrict μ (Ι a b)) h_bound : ∀ (n : ι), ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ι a b), ‖F n x‖ ≤ bound n x bound_summable : ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ι a b), Summable fun n => bound n x bound_integrable : IntegrableOn (fun t => ∑' (n : ι), bound n t) (Ι a b) h_lim : ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ι a b), HasSum (fun n => F n x) (f x) ⊢ HasSum (fun n => (if a ≤ b then 1 else -1) • ∫ (t : ℝ) in Ι a b, F n t ∂μ) ((if a ≤ b then 1 else -1) • ∫ (t : ℝ) in Ι a b, f t ∂μ) ** exact
(hasSum_integral_of_dominated_convergence bound hF_meas h_bound bound_summable bound_integrable
h_lim).const_smul
_ ** Qed
| |
intervalIntegral.continuousOn_primitive ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in Ioc a x, f t ∂μ) (Icc a b) ** by_cases h : a ≤ b ** case pos ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in Ioc a x, f t ∂μ) (Icc a b) ** have : ∀ x ∈ Icc a b, ∫ t in Ioc a x, f t ∂μ = ∫ t in a..x, f t ∂μ := by
intro x x_in
simp_rw [integral_of_le x_in.1] ** case pos ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b this : ∀ (x : ℝ), x ∈ Icc a b → ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in Ioc a x, f t ∂μ) (Icc a b) ** rw [continuousOn_congr this] ** case pos ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b this : ∀ (x : ℝ), x ∈ Icc a b → ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in a..x, f t ∂μ) (Icc a b) ** intro x₀ _ ** case pos ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b this : ∀ (x : ℝ), x ∈ Icc a b → ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ x₀ : ℝ a✝ : x₀ ∈ Icc a b ⊢ ContinuousWithinAt (fun x => ∫ (t : ℝ) in a..x, f t ∂μ) (Icc a b) x₀ ** refine' continuousWithinAt_primitive (measure_singleton x₀) _ ** case pos ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b this : ∀ (x : ℝ), x ∈ Icc a b → ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ x₀ : ℝ a✝ : x₀ ∈ Icc a b ⊢ IntervalIntegrable (fun t => f t) μ (min a a) (max a b) ** simp only [intervalIntegrable_iff_integrable_Ioc_of_le, min_eq_left, max_eq_right, h, min_self] ** case pos ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b this : ∀ (x : ℝ), x ∈ Icc a b → ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ x₀ : ℝ a✝ : x₀ ∈ Icc a b ⊢ IntegrableOn (fun t => f t) (Ioc a b) ** exact h_int.mono Ioc_subset_Icc_self le_rfl ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b ⊢ ∀ (x : ℝ), x ∈ Icc a b → ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ ** intro x x_in ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : a ≤ b x : ℝ x_in : x ∈ Icc a b ⊢ ∫ (t : ℝ) in Ioc a x, f t ∂μ = ∫ (t : ℝ) in a..x, f t ∂μ ** simp_rw [integral_of_le x_in.1] ** case neg ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : ¬a ≤ b ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in Ioc a x, f t ∂μ) (Icc a b) ** rw [Icc_eq_empty h] ** case neg ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f (Icc a b) h : ¬a ≤ b ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in Ioc a x, f t ∂μ) ∅ ** exact continuousOn_empty _ ** Qed
| |
intervalIntegral.continuousOn_primitive_interval' ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntervalIntegrable f μ b₁ b₂ ha : a ∈ [[b₁, b₂]] x✝¹ : ℝ x✝ : x✝¹ ∈ [[b₁, b₂]] ⊢ ContinuousWithinAt (fun b => ∫ (x : ℝ) in a..b, f x ∂μ) [[b₁, b₂]] x✝¹ ** refine continuousWithinAt_primitive (measure_singleton _) ?_ ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntervalIntegrable f μ b₁ b₂ ha : a ∈ [[b₁, b₂]] x✝¹ : ℝ x✝ : x✝¹ ∈ [[b₁, b₂]] ⊢ IntervalIntegrable (fun x => f x) μ (min a (b₁ ⊓ b₂)) (max a (b₁ ⊔ b₂)) ** rw [min_eq_right ha.1, max_eq_right ha.2] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntervalIntegrable f μ b₁ b₂ ha : a ∈ [[b₁, b₂]] x✝¹ : ℝ x✝ : x✝¹ ∈ [[b₁, b₂]] ⊢ IntervalIntegrable (fun x => f x) μ (b₁ ⊓ b₂) (b₁ ⊔ b₂) ** simpa [intervalIntegrable_iff, uIoc] using h_int ** Qed
| |
intervalIntegral.continuousOn_primitive_interval_left ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f [[a, b]] ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in x..b, f t ∂μ) [[a, b]] ** rw [uIcc_comm a b] at h_int ⊢ ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f [[b, a]] ⊢ ContinuousOn (fun x => ∫ (t : ℝ) in x..b, f t ∂μ) [[b, a]] ** simp only [integral_symm b] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : IntegrableOn f [[b, a]] ⊢ ContinuousOn (fun x => -∫ (t : ℝ) in b..x, f t ∂μ) [[b, a]] ** exact (continuousOn_primitive_interval h_int).neg ** Qed
| |
intervalIntegral.continuous_primitive ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a✝ b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : ∀ (a b : ℝ), IntervalIntegrable f μ a b a : ℝ ⊢ Continuous fun b => ∫ (x : ℝ) in a..b, f x ∂μ ** rw [continuous_iff_continuousAt] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a✝ b b₀ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : ∀ (a b : ℝ), IntervalIntegrable f μ a b a : ℝ ⊢ ∀ (x : ℝ), ContinuousAt (fun b => ∫ (x : ℝ) in a..b, f x ∂μ) x ** intro b₀ ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a✝ b b₀✝ b₁ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : ∀ (a b : ℝ), IntervalIntegrable f μ a b a b₀ : ℝ ⊢ ContinuousAt (fun b => ∫ (x : ℝ) in a..b, f x ∂μ) b₀ ** cases' exists_lt b₀ with b₁ hb₁ ** case intro ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a✝ b b₀✝ b₁✝ b₂ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : ∀ (a b : ℝ), IntervalIntegrable f μ a b a b₀ b₁ : ℝ hb₁ : b₁ < b₀ ⊢ ContinuousAt (fun b => ∫ (x : ℝ) in a..b, f x ∂μ) b₀ ** cases' exists_gt b₀ with b₂ hb₂ ** case intro.intro ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a✝ b b₀✝ b₁✝ b₂✝ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : ∀ (a b : ℝ), IntervalIntegrable f μ a b a b₀ b₁ : ℝ hb₁ : b₁ < b₀ b₂ : ℝ hb₂ : b₀ < b₂ ⊢ ContinuousAt (fun b => ∫ (x : ℝ) in a..b, f x ∂μ) b₀ ** apply ContinuousWithinAt.continuousAt _ (Icc_mem_nhds hb₁ hb₂) ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝³ : NormedAddCommGroup E inst✝² : CompleteSpace E inst✝¹ : NormedSpace ℝ E a✝ b b₀✝ b₁✝ b₂✝ : ℝ μ : Measure ℝ f g : ℝ → E inst✝ : NoAtoms μ h_int : ∀ (a b : ℝ), IntervalIntegrable f μ a b a b₀ b₁ : ℝ hb₁ : b₁ < b₀ b₂ : ℝ hb₂ : b₀ < b₂ ⊢ ContinuousWithinAt (fun b => ∫ (x : ℝ) in a..b, f x ∂μ) (Icc b₁ b₂) b₀ ** exact continuousWithinAt_primitive (measure_singleton b₀) (h_int _ _) ** Qed
| |
intervalIntegral.integral_eq_zero_iff_of_le_of_nonneg_ae ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : 0 ≤ᵐ[Measure.restrict μ (Ioc a b)] f hfi : IntervalIntegrable f μ a b ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ↔ f =ᵐ[Measure.restrict μ (Ioc a b)] 0 ** rw [integral_of_le hab, integral_eq_zero_iff_of_nonneg_ae hf hfi.1] ** Qed
| |
intervalIntegral.integral_eq_zero_iff_of_nonneg_ae ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ioc a b ∪ Ioc b a)] f hfi : IntervalIntegrable f μ a b ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ↔ f =ᵐ[Measure.restrict μ (Ioc a b ∪ Ioc b a)] 0 ** cases' le_total a b with hab hab <;>
simp only [Ioc_eq_empty hab.not_lt, empty_union, union_empty] at hf ⊢ ** case inl ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hfi : IntervalIntegrable f μ a b hab : a ≤ b hf : 0 ≤ᵐ[Measure.restrict μ (Ioc a b)] f ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ↔ f =ᵐ[Measure.restrict μ (Ioc a b)] 0 ** exact integral_eq_zero_iff_of_le_of_nonneg_ae hab hf hfi ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hfi : IntervalIntegrable f μ a b hab : b ≤ a hf : 0 ≤ᵐ[Measure.restrict μ (Ioc b a)] f ⊢ ∫ (x : ℝ) in a..b, f x ∂μ = 0 ↔ f =ᵐ[Measure.restrict μ (Ioc b a)] 0 ** rw [integral_symm, neg_eq_zero, integral_eq_zero_iff_of_le_of_nonneg_ae hab hf hfi.symm] ** Qed
| |
intervalIntegral.integral_pos_iff_support_of_nonneg_ae' ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ι a b)] f hfi : IntervalIntegrable f μ a b ⊢ 0 < ∫ (x : ℝ) in a..b, f x ∂μ ↔ a < b ∧ 0 < ↑↑μ (support f ∩ Ioc a b) ** cases' lt_or_le a b with hab hba ** case inl ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ι a b)] f hfi : IntervalIntegrable f μ a b hab : a < b ⊢ 0 < ∫ (x : ℝ) in a..b, f x ∂μ ↔ a < b ∧ 0 < ↑↑μ (support f ∩ Ioc a b) ** rw [uIoc_of_le hab.le] at hf ** case inl ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ioc a b)] f hfi : IntervalIntegrable f μ a b hab : a < b ⊢ 0 < ∫ (x : ℝ) in a..b, f x ∂μ ↔ a < b ∧ 0 < ↑↑μ (support f ∩ Ioc a b) ** simp only [hab, true_and_iff, integral_of_le hab.le,
set_integral_pos_iff_support_of_nonneg_ae hf hfi.1] ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ι a b)] f hfi : IntervalIntegrable f μ a b hba : b ≤ a ⊢ 0 < ∫ (x : ℝ) in a..b, f x ∂μ ↔ a < b ∧ 0 < ↑↑μ (support f ∩ Ioc a b) ** suffices (∫ x in a..b, f x ∂μ) ≤ 0 by simp only [this.not_lt, hba.not_lt, false_and_iff] ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ι a b)] f hfi : IntervalIntegrable f μ a b hba : b ≤ a ⊢ ∫ (x : ℝ) in a..b, f x ∂μ ≤ 0 ** rw [integral_of_ge hba, neg_nonpos] ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ι a b)] f hfi : IntervalIntegrable f μ a b hba : b ≤ a ⊢ 0 ≤ ∫ (x : ℝ) in Ioc b a, f x ∂μ ** rw [uIoc_comm, uIoc_of_le hba] at hf ** case inr ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ioc b a)] f hfi : IntervalIntegrable f μ a b hba : b ≤ a ⊢ 0 ≤ ∫ (x : ℝ) in Ioc b a, f x ∂μ ** exact integral_nonneg_of_ae hf ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hf : 0 ≤ᵐ[Measure.restrict μ (Ι a b)] f hfi : IntervalIntegrable f μ a b hba : b ≤ a this : ∫ (x : ℝ) in a..b, f x ∂μ ≤ 0 ⊢ 0 < ∫ (x : ℝ) in a..b, f x ∂μ ↔ a < b ∧ 0 < ↑↑μ (support f ∩ Ioc a b) ** simp only [this.not_lt, hba.not_lt, false_and_iff] ** Qed
| |
intervalIntegral.integral_lt_integral_of_ae_le_of_measure_setOf_lt_ne_zero ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hfi : IntervalIntegrable f μ a b hgi : IntervalIntegrable g μ a b hle : f ≤ᵐ[Measure.restrict μ (Ioc a b)] g hlt : ↑↑(Measure.restrict μ (Ioc a b)) {x | f x < g x} ≠ 0 ⊢ ∫ (x : ℝ) in a..b, f x ∂μ < ∫ (x : ℝ) in a..b, g x ∂μ ** rw [← sub_pos, ← integral_sub hgi hfi, integral_of_le hab,
MeasureTheory.integral_pos_iff_support_of_nonneg_ae] ** case hf ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hfi : IntervalIntegrable f μ a b hgi : IntervalIntegrable g μ a b hle : f ≤ᵐ[Measure.restrict μ (Ioc a b)] g hlt : ↑↑(Measure.restrict μ (Ioc a b)) {x | f x < g x} ≠ 0 ⊢ 0 ≤ᵐ[Measure.restrict μ (Ioc a b)] fun x => g x - f x case hfi ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hfi : IntervalIntegrable f μ a b hgi : IntervalIntegrable g μ a b hle : f ≤ᵐ[Measure.restrict μ (Ioc a b)] g hlt : ↑↑(Measure.restrict μ (Ioc a b)) {x | f x < g x} ≠ 0 ⊢ Integrable fun x => g x - f x ** exacts [hle.mono fun x => sub_nonneg.2, hgi.1.sub hfi.1] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hfi : IntervalIntegrable f μ a b hgi : IntervalIntegrable g μ a b hle : f ≤ᵐ[Measure.restrict μ (Ioc a b)] g hlt : ↑↑(Measure.restrict μ (Ioc a b)) {x | f x < g x} ≠ 0 ⊢ 0 < ↑↑(Measure.restrict μ (Ioc a b)) (support fun x => g x - f x) ** refine' pos_iff_ne_zero.2 (mt (measure_mono_null _) hlt) ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hfi : IntervalIntegrable f μ a b hgi : IntervalIntegrable g μ a b hle : f ≤ᵐ[Measure.restrict μ (Ioc a b)] g hlt : ↑↑(Measure.restrict μ (Ioc a b)) {x | f x < g x} ≠ 0 ⊢ {x | f x < g x} ⊆ support fun x => g x - f x ** exact fun x hx => (sub_pos.2 hx.out).ne' ** Qed
| |
intervalIntegral.integral_nonneg_of_ae_restrict ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : 0 ≤ᵐ[Measure.restrict μ (Icc a b)] f ⊢ 0 ≤ ∫ (u : ℝ) in a..b, f u ∂μ ** let H := ae_restrict_of_ae_restrict_of_subset Ioc_subset_Icc_self hf ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : 0 ≤ᵐ[Measure.restrict μ (Icc a b)] f H : ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ioc a b), OfNat.ofNat 0 x ≤ f x := ae_restrict_of_ae_restrict_of_subset Ioc_subset_Icc_self hf ⊢ 0 ≤ ∫ (u : ℝ) in a..b, f u ∂μ ** simpa only [integral_of_le hab] using set_integral_nonneg_of_ae_restrict H ** Qed
| |
intervalIntegral.abs_integral_le_integral_abs ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b ⊢ |∫ (x : ℝ) in a..b, f x ∂μ| ≤ ∫ (x : ℝ) in a..b, |f x| ∂μ ** simpa only [← Real.norm_eq_abs] using norm_integral_le_integral_norm hab ** Qed
| |
intervalIntegral.integral_mono_ae_restrict ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b h : f ≤ᵐ[Measure.restrict μ (Icc a b)] g ⊢ ∫ (u : ℝ) in a..b, f u ∂μ ≤ ∫ (u : ℝ) in a..b, g u ∂μ ** let H := h.filter_mono <| ae_mono <| Measure.restrict_mono Ioc_subset_Icc_self <| le_refl μ ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b h : f ≤ᵐ[Measure.restrict μ (Icc a b)] g H : ∀ᵐ (x : ℝ) ∂Measure.restrict μ (Ioc a b), f x ≤ g x := Eventually.filter_mono (ae_mono (Measure.restrict_mono Ioc_subset_Icc_self (le_refl μ))) h ⊢ ∫ (u : ℝ) in a..b, f u ∂μ ≤ ∫ (u : ℝ) in a..b, g u ∂μ ** simpa only [integral_of_le hab] using set_integral_mono_ae_restrict hf.1 hg.1 H ** Qed
| |
intervalIntegral.integral_mono_ae ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b h : f ≤ᵐ[μ] g ⊢ ∫ (u : ℝ) in a..b, f u ∂μ ≤ ∫ (u : ℝ) in a..b, g u ∂μ ** simpa only [integral_of_le hab] using set_integral_mono_ae hf.1 hg.1 h ** Qed
| |
intervalIntegral.integral_mono_on ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b h : ∀ (x : ℝ), x ∈ Icc a b → f x ≤ g x ⊢ ∫ (u : ℝ) in a..b, f u ∂μ ≤ ∫ (u : ℝ) in a..b, g u ∂μ ** let H x hx := h x <| Ioc_subset_Icc_self hx ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab : a ≤ b hf : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b h : ∀ (x : ℝ), x ∈ Icc a b → f x ≤ g x H : ∀ (x : ℝ), x ∈ Ioc a b → f x ≤ g x := fun x hx => h x (Ioc_subset_Icc_self hx) ⊢ ∫ (u : ℝ) in a..b, f u ∂μ ≤ ∫ (u : ℝ) in a..b, g u ∂μ ** simpa only [integral_of_le hab] using set_integral_mono_on hf.1 hg.1 measurableSet_Ioc H ** Qed
| |
intervalIntegral.integral_mono_interval ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab✝ : a ≤ b hf✝ : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b c d : ℝ hca : c ≤ a hab : a ≤ b hbd : b ≤ d hf : 0 ≤ᵐ[Measure.restrict μ (Ioc c d)] f hfi : IntervalIntegrable f μ c d ⊢ ∫ (x : ℝ) in a..b, f x ∂μ ≤ ∫ (x : ℝ) in c..d, f x ∂μ ** rw [integral_of_le hab, integral_of_le (hca.trans (hab.trans hbd))] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E f g : ℝ → ℝ a b : ℝ μ : Measure ℝ hab✝ : a ≤ b hf✝ : IntervalIntegrable f μ a b hg : IntervalIntegrable g μ a b c d : ℝ hca : c ≤ a hab : a ≤ b hbd : b ≤ d hf : 0 ≤ᵐ[Measure.restrict μ (Ioc c d)] f hfi : IntervalIntegrable f μ c d ⊢ ∫ (x : ℝ) in Ioc a b, f x ∂μ ≤ ∫ (x : ℝ) in Ioc c d, f x ∂μ ** exact set_integral_mono_set hfi.1 hf (Ioc_subset_Ioc hca hbd).eventuallyLE ** Qed
| |
MeasureTheory.Integrable.hasSum_intervalIntegral ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E μ : Measure ℝ f : ℝ → E hfi : Integrable f y : ℝ ⊢ HasSum (fun n => ∫ (x : ℝ) in y + ↑n..y + ↑n + 1, f x ∂μ) (∫ (x : ℝ), f x ∂μ) ** simp_rw [integral_of_le (le_add_of_nonneg_right zero_le_one)] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E μ : Measure ℝ f : ℝ → E hfi : Integrable f y : ℝ ⊢ HasSum (fun n => ∫ (x : ℝ) in Ioc (y + ↑n) (y + ↑n + 1), f x ∂μ) (∫ (x : ℝ), f x ∂μ) ** rw [← integral_univ, ← iUnion_Ioc_add_int_cast y] ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E μ : Measure ℝ f : ℝ → E hfi : Integrable f y : ℝ ⊢ HasSum (fun n => ∫ (x : ℝ) in Ioc (y + ↑n) (y + ↑n + 1), f x ∂μ) (∫ (x : ℝ) in ⋃ n, Ioc (y + ↑n) (y + ↑n + 1), f x ∂μ) ** exact
hasSum_integral_iUnion (fun i => measurableSet_Ioc) (pairwise_disjoint_Ioc_add_int_cast y)
hfi.integrableOn ** Qed
| |
MeasureTheory.Integrable.hasSum_intervalIntegral_comp_add_int ** ι : Type u_1 𝕜 : Type u_2 E : Type u_3 F : Type u_4 A : Type u_5 inst✝² : NormedAddCommGroup E inst✝¹ : CompleteSpace E inst✝ : NormedSpace ℝ E μ : Measure ℝ f : ℝ → E hfi : Integrable f ⊢ HasSum (fun n => ∫ (x : ℝ) in 0 ..1, f (x + ↑n)) (∫ (x : ℝ), f x) ** simpa only [integral_comp_add_right, zero_add, add_comm (1:ℝ)] using hfi.hasSum_intervalIntegral 0 ** Qed
| |
exp_neg_integrableOn_Ioi ** a b : ℝ h : 0 < b ⊢ IntegrableOn (fun x => rexp (-b * x)) (Ioi a) ** have : Tendsto (fun x => -exp (-b * x) / b) atTop (𝓝 (-0 / b)) := by
refine' Tendsto.div_const (Tendsto.neg _) _
exact tendsto_exp_atBot.comp (tendsto_id.neg_const_mul_atTop (Right.neg_neg_iff.2 h)) ** a b : ℝ h : 0 < b this : Tendsto (fun x => -rexp (-b * x) / b) atTop (𝓝 (-0 / b)) ⊢ IntegrableOn (fun x => rexp (-b * x)) (Ioi a) ** refine' integrableOn_Ioi_deriv_of_nonneg' (fun x _ => _) (fun x _ => (exp_pos _).le) this ** a b : ℝ h : 0 < b this : Tendsto (fun x => -rexp (-b * x) / b) atTop (𝓝 (-0 / b)) x : ℝ x✝ : x ∈ Ici a ⊢ HasDerivAt (fun x => -rexp (-b * x) / b) (rexp (-b * x)) x ** simpa [h.ne'] using ((hasDerivAt_id x).const_mul b).neg.exp.neg.div_const b ** a b : ℝ h : 0 < b ⊢ Tendsto (fun x => -rexp (-b * x) / b) atTop (𝓝 (-0 / b)) ** refine' Tendsto.div_const (Tendsto.neg _) _ ** a b : ℝ h : 0 < b ⊢ Tendsto (fun x => rexp (-b * x)) atTop (𝓝 0) ** exact tendsto_exp_atBot.comp (tendsto_id.neg_const_mul_atTop (Right.neg_neg_iff.2 h)) ** Qed
| |
MeasureTheory.FinMeasAdditive.zero ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β s t : Set α x✝⁴ : MeasurableSet s x✝³ : MeasurableSet t x✝² : ↑↑μ s ≠ ⊤ x✝¹ : ↑↑μ t ≠ ⊤ x✝ : s ∩ t = ∅ ⊢ OfNat.ofNat 0 (s ∪ t) = OfNat.ofNat 0 s + OfNat.ofNat 0 t ** simp ** Qed
| |
MeasureTheory.FinMeasAdditive.add ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β hT : FinMeasAdditive μ T hT' : FinMeasAdditive μ T' ⊢ FinMeasAdditive μ (T + T') ** intro s t hs ht hμs hμt hst ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β hT : FinMeasAdditive μ T hT' : FinMeasAdditive μ T' s t : Set α hs : MeasurableSet s ht : MeasurableSet t hμs : ↑↑μ s ≠ ⊤ hμt : ↑↑μ t ≠ ⊤ hst : s ∩ t = ∅ ⊢ (T + T') (s ∪ t) = (T + T') s + (T + T') t ** simp only [hT s t hs ht hμs hμt hst, hT' s t hs ht hμs hμt hst, Pi.add_apply] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β hT : FinMeasAdditive μ T hT' : FinMeasAdditive μ T' s t : Set α hs : MeasurableSet s ht : MeasurableSet t hμs : ↑↑μ s ≠ ⊤ hμt : ↑↑μ t ≠ ⊤ hst : s ∩ t = ∅ ⊢ T s + T t + (T' s + T' t) = T s + T' s + (T t + T' t) ** abel ** Qed
| |
MeasureTheory.FinMeasAdditive.smul ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁹ : NormedAddCommGroup E inst✝⁸ : NormedSpace ℝ E inst✝⁷ : NormedAddCommGroup F inst✝⁶ : NormedSpace ℝ F inst✝⁵ : NormedAddCommGroup F' inst✝⁴ : NormedSpace ℝ F' inst✝³ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝² : AddCommMonoid β T T' : Set α → β inst✝¹ : Monoid 𝕜 inst✝ : DistribMulAction 𝕜 β hT : FinMeasAdditive μ T c : 𝕜 s t : Set α hs : MeasurableSet s ht : MeasurableSet t hμs : ↑↑μ s ≠ ⊤ hμt : ↑↑μ t ≠ ⊤ hst : s ∩ t = ∅ ⊢ (fun s => c • T s) (s ∪ t) = (fun s => c • T s) s + (fun s => c • T s) t ** simp [hT s t hs ht hμs hμt hst] ** Qed
| |
MeasureTheory.FinMeasAdditive.of_smul_measure ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : FinMeasAdditive (c • μ) T ⊢ FinMeasAdditive μ T ** refine' of_eq_top_imp_eq_top (fun s _ hμs => _) hT ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : FinMeasAdditive (c • μ) T s : Set α x✝ : MeasurableSet s hμs : ↑↑(c • μ) s = ⊤ ⊢ ↑↑μ s = ⊤ ** rw [Measure.smul_apply, smul_eq_mul, ENNReal.mul_eq_top] at hμs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : FinMeasAdditive (c • μ) T s : Set α x✝ : MeasurableSet s hμs : c ≠ 0 ∧ ↑↑μ s = ⊤ ∨ c = ⊤ ∧ ↑↑μ s ≠ 0 ⊢ ↑↑μ s = ⊤ ** simp only [hc_ne_top, or_false_iff, Ne.def, false_and_iff] at hμs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : FinMeasAdditive (c • μ) T s : Set α x✝ : MeasurableSet s hμs : ¬c = 0 ∧ ↑↑μ s = ⊤ ⊢ ↑↑μ s = ⊤ ** exact hμs.2 ** Qed
| |
MeasureTheory.FinMeasAdditive.smul_measure ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_zero : c ≠ 0 hT : FinMeasAdditive μ T ⊢ FinMeasAdditive (c • μ) T ** refine' of_eq_top_imp_eq_top (fun s _ hμs => _) hT ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_zero : c ≠ 0 hT : FinMeasAdditive μ T s : Set α x✝ : MeasurableSet s hμs : ↑↑μ s = ⊤ ⊢ ↑↑(c • μ) s = ⊤ ** rw [Measure.smul_apply, smul_eq_mul, ENNReal.mul_eq_top] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_zero : c ≠ 0 hT : FinMeasAdditive μ T s : Set α x✝ : MeasurableSet s hμs : ↑↑μ s = ⊤ ⊢ c ≠ 0 ∧ ↑↑μ s = ⊤ ∨ c = ⊤ ∧ ↑↑μ s ≠ 0 ** simp only [hc_ne_zero, true_and_iff, Ne.def, not_false_iff] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T T' : Set α → β c : ℝ≥0∞ hc_ne_zero : c ≠ 0 hT : FinMeasAdditive μ T s : Set α x✝ : MeasurableSet s hμs : ↑↑μ s = ⊤ ⊢ ↑↑μ s = ⊤ ∨ c = ⊤ ∧ ¬↑↑μ s = 0 ** exact Or.inl hμs ** Qed
| |
MeasureTheory.FinMeasAdditive.map_iUnion_fin_meas_set_eq_sum ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) hSp : ∀ (i : ι), i ∈ sι → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ sι → ∀ (j : ι), j ∈ sι → i ≠ j → Disjoint (S i) (S j) ⊢ T (⋃ i ∈ sι, S i) = ∑ i in sι, T (S i) ** revert hSp h_disj ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) ⊢ (∀ (i : ι), i ∈ sι → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ sι → ∀ (j : ι), j ∈ sι → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ sι, S i) = ∑ i in sι, T (S i) ** refine' Finset.induction_on sι _ _ ** case refine'_2 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) ⊢ ∀ ⦃a : ι⦄ {s : Finset ι}, ¬a ∈ s → ((∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i)) → (∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ insert a s, S i) = ∑ i in insert a s, T (S i) ** intro a s has h hps h_disj ** case refine'_2 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ T (⋃ i ∈ insert a s, S i) = ∑ i in insert a s, T (S i) ** rw [Finset.sum_insert has, ← h] ** case refine'_2 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ T (⋃ i ∈ insert a s, S i) = T (S a) + T (⋃ i ∈ s, S i) case refine'_2.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤ case refine'_2.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j) ** swap ** case refine'_2 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ T (⋃ i ∈ insert a s, S i) = T (S a) + T (⋃ i ∈ s, S i) case refine'_2.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j) ** swap ** case refine'_2 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ T (⋃ i ∈ insert a s, S i) = T (S a) + T (⋃ i ∈ s, S i) ** rw [←
h_add (S a) (⋃ i ∈ s, S i) (hS_meas a) (measurableSet_biUnion _ fun i _ => hS_meas i)
(hps a (Finset.mem_insert_self a s))] ** case refine'_1 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) ⊢ (∀ (i : ι), i ∈ ∅ → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ ∅ → ∀ (j : ι), j ∈ ∅ → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ ∅, S i) = ∑ i in ∅, T (S i) ** simp only [Finset.not_mem_empty, IsEmpty.forall_iff, iUnion_false, iUnion_empty, sum_empty,
forall₂_true_iff, imp_true_iff, forall_true_left, not_false_iff, T_empty] ** case refine'_2.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤ ** exact fun i hi => hps i (Finset.mem_insert_of_mem hi) ** case refine'_2.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j) ** exact fun i hi j hj hij =>
h_disj i (Finset.mem_insert_of_mem hi) j (Finset.mem_insert_of_mem hj) hij ** case refine'_2 α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ T (⋃ i ∈ insert a s, S i) = T (S a ∪ ⋃ i ∈ s, S i) ** congr ** case refine'_2.e_a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ⋃ i ∈ insert a s, S i = S a ∪ ⋃ i ∈ s, S i ** convert Finset.iSup_insert a s S ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ↑↑μ (⋃ i ∈ s, S i) ≠ ⊤ ** exact
((measure_biUnion_finset_le _ _).trans_lt <|
ENNReal.sum_lt_top fun i hi => hps i <| Finset.mem_insert_of_mem hi).ne ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ S a ∩ ⋃ i ∈ s, S i = ∅ ** simp_rw [Set.inter_iUnion] ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) ⊢ ⋃ i ∈ s, S a ∩ S i = ∅ ** refine' iUnion_eq_empty.mpr fun i => iUnion_eq_empty.mpr fun hi => _ ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) i : ι hi : i ∈ s ⊢ S a ∩ S i = ∅ ** rw [← Set.disjoint_iff_inter_eq_empty] ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) i : ι hi : i ∈ s ⊢ Disjoint (S a) (S i) ** refine' h_disj a (Finset.mem_insert_self a s) i (Finset.mem_insert_of_mem hi) fun hai => _ ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) i : ι hi : i ∈ s hai : a = i ⊢ False ** rw [← hai] at hi ** case refine'_2.a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : AddCommMonoid β T✝ T' T : Set α → β T_empty : T ∅ = 0 h_add : FinMeasAdditive μ T ι : Type u_8 S : ι → Set α sι : Finset ι hS_meas : ∀ (i : ι), MeasurableSet (S i) a : ι s : Finset ι has : ¬a ∈ s h : (∀ (i : ι), i ∈ s → ↑↑μ (S i) ≠ ⊤) → (∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → i ≠ j → Disjoint (S i) (S j)) → T (⋃ i ∈ s, S i) = ∑ i in s, T (S i) hps : ∀ (i : ι), i ∈ insert a s → ↑↑μ (S i) ≠ ⊤ h_disj : ∀ (i : ι), i ∈ insert a s → ∀ (j : ι), j ∈ insert a s → i ≠ j → Disjoint (S i) (S j) i : ι hi : a ∈ s hai : a = i ⊢ False ** exact has hi ** Qed
| |
MeasureTheory.DominatedFinMeasAdditive.eq_zero_of_measure_zero ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β✝ : Type u_7 inst✝¹ : SeminormedAddCommGroup β✝ T✝ T' : Set α → β✝ C✝ C' : ℝ β : Type u_8 inst✝ : NormedAddCommGroup β T : Set α → β C : ℝ hT : DominatedFinMeasAdditive μ T C s : Set α hs : MeasurableSet s hs_zero : ↑↑μ s = 0 ⊢ T s = 0 ** refine' norm_eq_zero.mp _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β✝ : Type u_7 inst✝¹ : SeminormedAddCommGroup β✝ T✝ T' : Set α → β✝ C✝ C' : ℝ β : Type u_8 inst✝ : NormedAddCommGroup β T : Set α → β C : ℝ hT : DominatedFinMeasAdditive μ T C s : Set α hs : MeasurableSet s hs_zero : ↑↑μ s = 0 ⊢ ‖T s‖ = 0 ** refine' ((hT.2 s hs (by simp [hs_zero])).trans (le_of_eq _)).antisymm (norm_nonneg _) ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β✝ : Type u_7 inst✝¹ : SeminormedAddCommGroup β✝ T✝ T' : Set α → β✝ C✝ C' : ℝ β : Type u_8 inst✝ : NormedAddCommGroup β T : Set α → β C : ℝ hT : DominatedFinMeasAdditive μ T C s : Set α hs : MeasurableSet s hs_zero : ↑↑μ s = 0 ⊢ C * ENNReal.toReal (↑↑μ s) = 0 ** rw [hs_zero, ENNReal.zero_toReal, mul_zero] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β✝ : Type u_7 inst✝¹ : SeminormedAddCommGroup β✝ T✝ T' : Set α → β✝ C✝ C' : ℝ β : Type u_8 inst✝ : NormedAddCommGroup β T : Set α → β C : ℝ hT : DominatedFinMeasAdditive μ T C s : Set α hs : MeasurableSet s hs_zero : ↑↑μ s = 0 ⊢ ↑↑μ s < ⊤ ** simp [hs_zero] ** Qed
| |
MeasureTheory.DominatedFinMeasAdditive.of_measure_le ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C ⊢ DominatedFinMeasAdditive μ' T C ** have h' : ∀ s, MeasurableSet s → μ s = ∞ → μ' s = ∞ := by
intro s hs hμs; rw [eq_top_iff, ← hμs]; exact h s hs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C h' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = ⊤ → ↑↑μ' s = ⊤ ⊢ DominatedFinMeasAdditive μ' T C ** refine' ⟨hT.1.of_eq_top_imp_eq_top h', fun s hs hμ's => _⟩ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C h' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = ⊤ → ↑↑μ' s = ⊤ s : Set α hs : MeasurableSet s hμ's : ↑↑μ' s < ⊤ ⊢ ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ' s) ** have hμs : μ s < ∞ := (h s hs).trans_lt hμ's ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C h' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = ⊤ → ↑↑μ' s = ⊤ s : Set α hs : MeasurableSet s hμ's : ↑↑μ' s < ⊤ hμs : ↑↑μ s < ⊤ ⊢ ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ' s) ** refine' (hT.2 s hs hμs).trans (mul_le_mul le_rfl _ ENNReal.toReal_nonneg hC) ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C h' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = ⊤ → ↑↑μ' s = ⊤ s : Set α hs : MeasurableSet s hμ's : ↑↑μ' s < ⊤ hμs : ↑↑μ s < ⊤ ⊢ ENNReal.toReal (↑↑μ s) ≤ ENNReal.toReal (↑↑μ' s) ** rw [toReal_le_toReal hμs.ne hμ's.ne] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C h' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = ⊤ → ↑↑μ' s = ⊤ s : Set α hs : MeasurableSet s hμ's : ↑↑μ' s < ⊤ hμs : ↑↑μ s < ⊤ ⊢ ↑↑μ s ≤ ↑↑μ' s ** exact h s hs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C ⊢ ∀ (s : Set α), MeasurableSet s → ↑↑μ s = ⊤ → ↑↑μ' s = ⊤ ** intro s hs hμs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C s : Set α hs : MeasurableSet s hμs : ↑↑μ s = ⊤ ⊢ ↑↑μ' s = ⊤ ** rw [eq_top_iff, ← hμs] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ μ' : Measure α h : μ ≤ μ' hT : DominatedFinMeasAdditive μ T C hC : 0 ≤ C s : Set α hs : MeasurableSet s hμs : ↑↑μ s = ⊤ ⊢ ↑↑μ s ≤ ↑↑μ' s ** exact h s hs ** Qed
| |
MeasureTheory.DominatedFinMeasAdditive.of_smul_measure ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C ⊢ DominatedFinMeasAdditive μ T (ENNReal.toReal c * C) ** have h : ∀ s, MeasurableSet s → c • μ s = ∞ → μ s = ∞ := by
intro s _ hcμs
simp only [hc_ne_top, Algebra.id.smul_eq_mul, ENNReal.mul_eq_top, or_false_iff, Ne.def,
false_and_iff] at hcμs
exact hcμs.2 ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C h : ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ ⊢ DominatedFinMeasAdditive μ T (ENNReal.toReal c * C) ** refine' ⟨hT.1.of_eq_top_imp_eq_top (μ := c • μ) h, fun s hs hμs => _⟩ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C h : ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ s : Set α hs : MeasurableSet s hμs : ↑↑μ s < ⊤ ⊢ ‖T s‖ ≤ ENNReal.toReal c * C * ENNReal.toReal (↑↑μ s) ** have hcμs : c • μ s ≠ ∞ := mt (h s hs) hμs.ne ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C h : ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ s : Set α hs : MeasurableSet s hμs : ↑↑μ s < ⊤ hcμs : c • ↑↑μ s ≠ ⊤ ⊢ ‖T s‖ ≤ ENNReal.toReal c * C * ENNReal.toReal (↑↑μ s) ** rw [smul_eq_mul] at hcμs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C h : ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ s : Set α hs : MeasurableSet s hμs : ↑↑μ s < ⊤ hcμs : c * ↑↑μ s ≠ ⊤ ⊢ ‖T s‖ ≤ ENNReal.toReal c * C * ENNReal.toReal (↑↑μ s) ** simp_rw [DominatedFinMeasAdditive, Measure.smul_apply, smul_eq_mul, toReal_mul] at hT ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ h : ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ s : Set α hs : MeasurableSet s hμs : ↑↑μ s < ⊤ hcμs : c * ↑↑μ s ≠ ⊤ hT : FinMeasAdditive (c • μ) T ∧ ∀ (s : Set α), MeasurableSet s → c * ↑↑μ s < ⊤ → ‖T s‖ ≤ C * (ENNReal.toReal c * ENNReal.toReal (↑↑μ s)) ⊢ ‖T s‖ ≤ ENNReal.toReal c * C * ENNReal.toReal (↑↑μ s) ** refine' (hT.2 s hs hcμs.lt_top).trans (le_of_eq _) ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ h : ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ s : Set α hs : MeasurableSet s hμs : ↑↑μ s < ⊤ hcμs : c * ↑↑μ s ≠ ⊤ hT : FinMeasAdditive (c • μ) T ∧ ∀ (s : Set α), MeasurableSet s → c * ↑↑μ s < ⊤ → ‖T s‖ ≤ C * (ENNReal.toReal c * ENNReal.toReal (↑↑μ s)) ⊢ C * (ENNReal.toReal c * ENNReal.toReal (↑↑μ s)) = ENNReal.toReal c * C * ENNReal.toReal (↑↑μ s) ** ring ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C ⊢ ∀ (s : Set α), MeasurableSet s → c • ↑↑μ s = ⊤ → ↑↑μ s = ⊤ ** intro s _ hcμs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C s : Set α a✝ : MeasurableSet s hcμs : c • ↑↑μ s = ⊤ ⊢ ↑↑μ s = ⊤ ** simp only [hc_ne_top, Algebra.id.smul_eq_mul, ENNReal.mul_eq_top, or_false_iff, Ne.def,
false_and_iff] at hcμs ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁷ : NormedAddCommGroup E inst✝⁶ : NormedSpace ℝ E inst✝⁵ : NormedAddCommGroup F inst✝⁴ : NormedSpace ℝ F inst✝³ : NormedAddCommGroup F' inst✝² : NormedSpace ℝ F' inst✝¹ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α β : Type u_7 inst✝ : SeminormedAddCommGroup β T T' : Set α → β C C' : ℝ c : ℝ≥0∞ hc_ne_top : c ≠ ⊤ hT : DominatedFinMeasAdditive (c • μ) T C s : Set α a✝ : MeasurableSet s hcμs : ¬c = 0 ∧ ↑↑μ s = ⊤ ⊢ ↑↑μ s = ⊤ ** exact hcμs.2 ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_zero ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α f : α →ₛ F ⊢ setToSimpleFunc 0 f = 0 ** simp [setToSimpleFunc] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_zero' ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = 0 f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T f = 0 ** simp_rw [setToSimpleFunc] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = 0 f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) x = 0 ** refine' sum_eq_zero fun x _ => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = 0 f : α →ₛ E hf : Integrable ↑f x : E x✝ : x ∈ SimpleFunc.range f ⊢ ↑(T (↑f ⁻¹' {x})) x = 0 ** by_cases hx0 : x = 0 ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = 0 f : α →ₛ E hf : Integrable ↑f x : E x✝ : x ∈ SimpleFunc.range f hx0 : ¬x = 0 ⊢ ↑(T (↑f ⁻¹' {x})) x = 0 ** rw [h_zero (f ⁻¹' ({x} : Set E)) (measurableSet_fiber _ _)
(measure_preimage_lt_top_of_integrable f hf hx0),
ContinuousLinearMap.zero_apply] ** case pos α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = 0 f : α →ₛ E hf : Integrable ↑f x : E x✝ : x ∈ SimpleFunc.range f hx0 : x = 0 ⊢ ↑(T (↑f ⁻¹' {x})) x = 0 ** simp [hx0] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_zero_apply ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F →L[ℝ] F' ⊢ setToSimpleFunc T 0 = 0 ** cases isEmpty_or_nonempty α <;> simp [setToSimpleFunc] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_eq_sum_filter ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F →L[ℝ] F' f : α →ₛ F ⊢ setToSimpleFunc T f = ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) x ** symm ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F →L[ℝ] F' f : α →ₛ F ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) x = setToSimpleFunc T f ** refine' sum_filter_of_ne fun x _ => mt fun hx0 => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F →L[ℝ] F' f : α →ₛ F x : F x✝ : x ∈ SimpleFunc.range f hx0 : x = 0 ⊢ ↑(T (↑f ⁻¹' {x})) x = 0 ** rw [hx0] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F →L[ℝ] F' f : α →ₛ F x : F x✝ : x ∈ SimpleFunc.range f hx0 : x = 0 ⊢ ↑(T (↑f ⁻¹' {0})) 0 = 0 ** exact ContinuousLinearMap.map_zero _ ** Qed
| |
MeasureTheory.SimpleFunc.map_setToSimpleFunc ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 ⊢ setToSimpleFunc T (map g f) = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (g x) ** have T_empty : T ∅ = 0 := h_add.map_empty_eq_zero ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 ⊢ setToSimpleFunc T (map g f) = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (g x) ** have hfp : ∀ x ∈ f.range, x ≠ 0 → μ (f ⁻¹' {x}) ≠ ∞ := fun x _ hx0 =>
(measure_preimage_lt_top_of_integrable f hf hx0).ne ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ ⊢ setToSimpleFunc T (map g f) = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (g x) ** simp only [setToSimpleFunc, range_map] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ ⊢ ∑ x in Finset.image g (SimpleFunc.range f), ↑(T (↑(map g f) ⁻¹' {x})) x = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (g x) ** refine' Finset.sum_image' _ fun b hb => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ b : G hb : b ∈ SimpleFunc.range f ⊢ ↑(T (↑(map g f) ⁻¹' {g b})) (g b) = ∑ x in filter (fun c' => g c' = g b) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** rcases mem_range.1 hb with ⟨a, rfl⟩ ** case intro α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f ⊢ ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** by_cases h0 : g (f a) = 0 ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 ⊢ ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** have h_left_eq :
T (map g f ⁻¹' {g (f a)}) (g (f a)) =
T (f ⁻¹' (f.range.filter fun b => g b = g (f a))) (g (f a)) :=
by congr; rw [map_preimage_singleton] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) ⊢ ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** rw [h_left_eq] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) ⊢ ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** have h_left_eq' :
T (f ⁻¹' (filter (fun b : G => g b = g (f a)) f.range)) (g (f a)) =
T (⋃ y ∈ filter (fun b : G => g b = g (f a)) f.range, f ⁻¹' {y}) (g (f a)) :=
by congr; rw [← Finset.set_biUnion_preimage_singleton] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** rw [h_left_eq'] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** rw [h_add.map_iUnion_fin_meas_set_eq_sum T T_empty] ** case pos α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : g (↑f a) = 0 ⊢ ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** simp_rw [h0] ** case pos α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : g (↑f a) = 0 ⊢ ↑(T (↑(map g f) ⁻¹' {0})) 0 = ∑ x in filter (fun c' => g c' = 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** rw [ContinuousLinearMap.map_zero, Finset.sum_eq_zero fun x hx => ?_] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : g (↑f a) = 0 x : G hx : x ∈ filter (fun c' => g c' = 0) (SimpleFunc.range f) ⊢ ↑(T (↑f ⁻¹' {x})) (g x) = 0 ** rw [mem_filter] at hx ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : g (↑f a) = 0 x : G hx : x ∈ SimpleFunc.range f ∧ g x = 0 ⊢ ↑(T (↑f ⁻¹' {x})) (g x) = 0 ** rw [hx.2, ContinuousLinearMap.map_zero] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 ⊢ ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) ** congr ** case e_a.e_a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 ⊢ ↑(map g f) ⁻¹' {g (↑f a)} = ↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)) ** rw [map_preimage_singleton] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) ⊢ ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ** congr ** case e_a.e_a α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) ⊢ ↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)) = ⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y} ** rw [← Finset.set_biUnion_preimage_singleton] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ↑(∑ i in filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), T (↑f ⁻¹' {i})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** simp only [sum_apply, ContinuousLinearMap.coe_sum'] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ∑ c in filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {c})) (g (↑f a)) = ∑ x in filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) (g x) ** refine' Finset.sum_congr rfl fun x hx => _ ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) x : G hx : x ∈ filter (fun c' => g c' = g (↑f a)) (SimpleFunc.range f) ⊢ ↑(T (↑f ⁻¹' {x})) (g (↑f a)) = ↑(T (↑f ⁻¹' {x})) (g x) ** rw [mem_filter] at hx ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) x : G hx : x ∈ SimpleFunc.range f ∧ g x = g (↑f a) ⊢ ↑(T (↑f ⁻¹' {x})) (g (↑f a)) = ↑(T (↑f ⁻¹' {x})) (g x) ** rw [hx.2] ** case neg.hS_meas α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ∀ (i : G), MeasurableSet (↑f ⁻¹' {i}) ** exact fun i => measurableSet_fiber _ _ ** case neg.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ∀ (i : G), i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) → ↑↑μ (↑f ⁻¹' {i}) ≠ ⊤ ** intro i hi ** case neg.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G hi : i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) ⊢ ↑↑μ (↑f ⁻¹' {i}) ≠ ⊤ ** rw [mem_filter] at hi ** case neg.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G hi : i ∈ SimpleFunc.range f ∧ g i = g (↑f a) ⊢ ↑↑μ (↑f ⁻¹' {i}) ≠ ⊤ ** refine' hfp i hi.1 fun hi0 => _ ** case neg.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G hi : i ∈ SimpleFunc.range f ∧ g i = g (↑f a) hi0 : i = 0 ⊢ False ** rw [hi0, hg] at hi ** case neg.hSp α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G hi : 0 ∈ SimpleFunc.range f ∧ 0 = g (↑f a) hi0 : i = 0 ⊢ False ** exact h0 hi.2.symm ** case neg.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) ⊢ ∀ (i : G), i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) → ∀ (j : G), j ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) → i ≠ j → Disjoint (↑f ⁻¹' {i}) (↑f ⁻¹' {j}) ** intro i _j hi _ hij ** case neg.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G _j : i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hi : G a✝ : hi ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hij : i ≠ hi ⊢ Disjoint (↑f ⁻¹' {i}) (↑f ⁻¹' {hi}) ** rw [Set.disjoint_iff] ** case neg.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G _j : i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hi : G a✝ : hi ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hij : i ≠ hi ⊢ ↑f ⁻¹' {i} ∩ ↑f ⁻¹' {hi} ⊆ ∅ ** intro x hx ** case neg.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G _j : i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hi : G a✝ : hi ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hij : i ≠ hi x : α hx : x ∈ ↑f ⁻¹' {i} ∩ ↑f ⁻¹' {hi} ⊢ x ∈ ∅ ** rw [Set.mem_inter_iff, Set.mem_preimage, Set.mem_preimage, Set.mem_singleton_iff,
Set.mem_singleton_iff] at hx ** case neg.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G _j : i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hi : G a✝ : hi ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hij : i ≠ hi x : α hx : ↑f x = i ∧ ↑f x = hi ⊢ x ∈ ∅ ** rw [← hx.1, ← hx.2] at hij ** case neg.h_disj α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' h_add : FinMeasAdditive μ T f : α →ₛ G hf : Integrable ↑f g : G → F hg : g 0 = 0 T_empty : T ∅ = 0 hfp : ∀ (x : G), x ∈ SimpleFunc.range f → x ≠ 0 → ↑↑μ (↑f ⁻¹' {x}) ≠ ⊤ a : α hb : ↑f a ∈ SimpleFunc.range f h0 : ¬g (↑f a) = 0 h_left_eq : ↑(T (↑(map g f) ⁻¹' {g (↑f a)})) (g (↑f a)) = ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) h_left_eq' : ↑(T (↑f ⁻¹' ↑(filter (fun b => g b = g (↑f a)) (SimpleFunc.range f)))) (g (↑f a)) = ↑(T (⋃ y ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f), ↑f ⁻¹' {y})) (g (↑f a)) i : G _j : i ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) hi : G a✝ : hi ∈ filter (fun b => g b = g (↑f a)) (SimpleFunc.range f) x : α hij : ↑f x ≠ ↑f x hx : ↑f x = i ∧ ↑f x = hi ⊢ x ∈ ∅ ** exact absurd rfl hij ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_congr_left ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F h : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = T' s f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T f = setToSimpleFunc T' f ** simp_rw [setToSimpleFunc] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F h : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = T' s f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) x = ∑ x in SimpleFunc.range f, ↑(T' (↑f ⁻¹' {x})) x ** refine' sum_congr rfl fun x _ => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F h : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = T' s f : α →ₛ E hf : Integrable ↑f x : E x✝ : x ∈ SimpleFunc.range f ⊢ ↑(T (↑f ⁻¹' {x})) x = ↑(T' (↑f ⁻¹' {x})) x ** by_cases hx0 : x = 0 ** case pos α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F h : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = T' s f : α →ₛ E hf : Integrable ↑f x : E x✝ : x ∈ SimpleFunc.range f hx0 : x = 0 ⊢ ↑(T (↑f ⁻¹' {x})) x = ↑(T' (↑f ⁻¹' {x})) x ** simp [hx0] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F h : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T s = T' s f : α →ₛ E hf : Integrable ↑f x : E x✝ : x ∈ SimpleFunc.range f hx0 : ¬x = 0 ⊢ ↑(T (↑f ⁻¹' {x})) x = ↑(T' (↑f ⁻¹' {x})) x ** rw [h (f ⁻¹' {x}) (SimpleFunc.measurableSet_fiber _ _)
(SimpleFunc.measure_preimage_lt_top_of_integrable _ hf hx0)] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_add_left ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T T' : Set α → F →L[ℝ] F' f : α →ₛ F ⊢ setToSimpleFunc (T + T') f = setToSimpleFunc T f + setToSimpleFunc T' f ** simp_rw [setToSimpleFunc, Pi.add_apply] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T T' : Set α → F →L[ℝ] F' f : α →ₛ F ⊢ ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x})) x = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) x + ∑ x in SimpleFunc.range f, ↑(T' (↑f ⁻¹' {x})) x ** push_cast ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T T' : Set α → F →L[ℝ] F' f : α →ₛ F ⊢ ∑ x in SimpleFunc.range f, (↑(T (↑f ⁻¹' {x})) + ↑(T' (↑f ⁻¹' {x}))) x = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) x + ∑ x in SimpleFunc.range f, ↑(T' (↑f ⁻¹' {x})) x ** simp_rw [Pi.add_apply, sum_add_distrib] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_add_left' ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T'' f = setToSimpleFunc T f + setToSimpleFunc T' f ** simp_rw [setToSimpleFunc_eq_sum_filter] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T'' (↑f ⁻¹' {x})) x = ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) x + ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T' (↑f ⁻¹' {x})) x ** suffices
∀ x ∈ filter (fun x : E => x ≠ 0) f.range, T'' (f ⁻¹' {x}) = T (f ⁻¹' {x}) + T' (f ⁻¹' {x}) by
rw [← sum_add_distrib]
refine' Finset.sum_congr rfl fun x hx => _
rw [this x hx]
push_cast
rw [Pi.add_apply] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f ⊢ ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) ** intro x hx ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) ** refine'
h_add (f ⁻¹' {x}) (measurableSet_preimage _ _) (measure_preimage_lt_top_of_integrable _ hf _) ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ x ≠ 0 ** rw [mem_filter] at hx ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f x : E hx : x ∈ SimpleFunc.range f ∧ x ≠ 0 ⊢ x ≠ 0 ** exact hx.2 ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T'' (↑f ⁻¹' {x})) x = ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) x + ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T' (↑f ⁻¹' {x})) x ** rw [← sum_add_distrib] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T'' (↑f ⁻¹' {x})) x = ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), (↑(T (↑f ⁻¹' {x})) x + ↑(T' (↑f ⁻¹' {x})) x) ** refine' Finset.sum_congr rfl fun x hx => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ ↑(T'' (↑f ⁻¹' {x})) x = ↑(T (↑f ⁻¹' {x})) x + ↑(T' (↑f ⁻¹' {x})) x ** rw [this x hx] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ ↑(T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x})) x = ↑(T (↑f ⁻¹' {x})) x + ↑(T' (↑f ⁻¹' {x})) x ** push_cast ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' T'' : Set α → E →L[ℝ] F h_add : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T'' s = T s + T' s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T'' (↑f ⁻¹' {x}) = T (↑f ⁻¹' {x}) + T' (↑f ⁻¹' {x}) x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ (↑(T (↑f ⁻¹' {x})) + ↑(T' (↑f ⁻¹' {x}))) x = ↑(T (↑f ⁻¹' {x})) x + ↑(T' (↑f ⁻¹' {x})) x ** rw [Pi.add_apply] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_smul_left ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F →L[ℝ] F' c : ℝ f : α →ₛ F ⊢ setToSimpleFunc (fun s => c • T s) f = c • setToSimpleFunc T f ** simp_rw [setToSimpleFunc, ContinuousLinearMap.smul_apply, smul_sum] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_smul_left' ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T' f = c • setToSimpleFunc T f ** simp_rw [setToSimpleFunc_eq_sum_filter] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T' (↑f ⁻¹' {x})) x = c • ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) x ** suffices ∀ x ∈ filter (fun x : E => x ≠ 0) f.range, T' (f ⁻¹' {x}) = c • T (f ⁻¹' {x}) by
rw [smul_sum]
refine' Finset.sum_congr rfl fun x hx => _
rw [this x hx]
rfl ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f ⊢ ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T' (↑f ⁻¹' {x}) = c • T (↑f ⁻¹' {x}) ** intro x hx ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ T' (↑f ⁻¹' {x}) = c • T (↑f ⁻¹' {x}) ** refine'
h_smul (f ⁻¹' {x}) (measurableSet_preimage _ _) (measure_preimage_lt_top_of_integrable _ hf _) ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ x ≠ 0 ** rw [mem_filter] at hx ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f x : E hx : x ∈ SimpleFunc.range f ∧ x ≠ 0 ⊢ x ≠ 0 ** exact hx.2 ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T' (↑f ⁻¹' {x}) = c • T (↑f ⁻¹' {x}) ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T' (↑f ⁻¹' {x})) x = c • ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T (↑f ⁻¹' {x})) x ** rw [smul_sum] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T' (↑f ⁻¹' {x}) = c • T (↑f ⁻¹' {x}) ⊢ ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), ↑(T' (↑f ⁻¹' {x})) x = ∑ x in filter (fun x => x ≠ 0) (SimpleFunc.range f), c • ↑(T (↑f ⁻¹' {x})) x ** refine' Finset.sum_congr rfl fun x hx => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T' (↑f ⁻¹' {x}) = c • T (↑f ⁻¹' {x}) x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ ↑(T' (↑f ⁻¹' {x})) x = c • ↑(T (↑f ⁻¹' {x})) x ** rw [this x hx] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T T' : Set α → E →L[ℝ] F' c : ℝ h_smul : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → T' s = c • T s f : α →ₛ E hf : Integrable ↑f this : ∀ (x : E), x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) → T' (↑f ⁻¹' {x}) = c • T (↑f ⁻¹' {x}) x : E hx : x ∈ filter (fun x => x ≠ 0) (SimpleFunc.range f) ⊢ ↑(c • T (↑f ⁻¹' {x})) x = c • ↑(T (↑f ⁻¹' {x})) x ** rfl ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_add ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : Integrable ↑g hp_pair : Integrable ↑(pair f g) ⊢ setToSimpleFunc T (f + g) = ∑ x in SimpleFunc.range (pair f g), ↑(T (↑(pair f g) ⁻¹' {x})) (x.1 + x.2) ** rw [add_eq_map₂, map_setToSimpleFunc T h_add hp_pair] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : Integrable ↑g hp_pair : Integrable ↑(pair f g) ⊢ 0.1 + 0.2 = 0 ** simp ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : Integrable ↑g hp_pair : Integrable ↑(pair f g) ⊢ ∑ x in SimpleFunc.range (pair f g), (↑(T (↑(pair f g) ⁻¹' {x})) x.1 + ↑(T (↑(pair f g) ⁻¹' {x})) x.2) = ∑ x in SimpleFunc.range (pair f g), ↑(T (↑(pair f g) ⁻¹' {x})) x.1 + ∑ x in SimpleFunc.range (pair f g), ↑(T (↑(pair f g) ⁻¹' {x})) x.2 ** rw [Finset.sum_add_distrib] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : Integrable ↑g hp_pair : Integrable ↑(pair f g) ⊢ ∑ x in SimpleFunc.range (pair f g), ↑(T (↑(pair f g) ⁻¹' {x})) x.1 + ∑ x in SimpleFunc.range (pair f g), ↑(T (↑(pair f g) ⁻¹' {x})) x.2 = setToSimpleFunc T (map Prod.fst (pair f g)) + setToSimpleFunc T (map Prod.snd (pair f g)) ** rw [map_setToSimpleFunc T h_add hp_pair Prod.snd_zero,
map_setToSimpleFunc T h_add hp_pair Prod.fst_zero] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_neg ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T (map Neg.neg f) = -setToSimpleFunc T f ** rw [map_setToSimpleFunc T h_add hf neg_zero, setToSimpleFunc, ← sum_neg_distrib] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (-x) = ∑ x in SimpleFunc.range f, -↑(T (↑f ⁻¹' {x})) x ** exact Finset.sum_congr rfl fun x _ => ContinuousLinearMap.map_neg _ _ ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_sub ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : Integrable ↑g ⊢ setToSimpleFunc T (f - g) = setToSimpleFunc T f - setToSimpleFunc T g ** rw [sub_eq_add_neg, setToSimpleFunc_add T h_add hf, setToSimpleFunc_neg T h_add hg,
sub_eq_add_neg] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : Integrable ↑g ⊢ Integrable ↑(-g) ** rw [integrable_iff] at hg ⊢ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : ∀ (y : E), y ≠ 0 → ↑↑μ (↑g ⁻¹' {y}) < ⊤ ⊢ ∀ (y : E), y ≠ 0 → ↑↑μ (↑(-g) ⁻¹' {y}) < ⊤ ** intro x hx_ne ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : ∀ (y : E), y ≠ 0 → ↑↑μ (↑g ⁻¹' {y}) < ⊤ x : E hx_ne : x ≠ 0 ⊢ ↑↑μ (↑(-g) ⁻¹' {x}) < ⊤ ** change μ (Neg.neg ∘ g ⁻¹' {x}) < ∞ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : ∀ (y : E), y ≠ 0 → ↑↑μ (↑g ⁻¹' {y}) < ⊤ x : E hx_ne : x ≠ 0 ⊢ ↑↑μ (Neg.neg ∘ ↑g ⁻¹' {x}) < ⊤ ** rw [preimage_comp, neg_preimage, Set.neg_singleton] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : ∀ (y : E), y ≠ 0 → ↑↑μ (↑g ⁻¹' {y}) < ⊤ x : E hx_ne : x ≠ 0 ⊢ ↑↑μ (↑g ⁻¹' {-x}) < ⊤ ** refine' hg (-x) _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T f g : α →ₛ E hf : Integrable ↑f hg : ∀ (y : E), y ≠ 0 → ↑↑μ (↑g ⁻¹' {y}) < ⊤ x : E hx_ne : x ≠ 0 ⊢ -x ≠ 0 ** simp [hx_ne] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_smul_real ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T c : ℝ f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T (c • f) = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (c • x) ** rw [smul_eq_map c f, map_setToSimpleFunc T h_add hf] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T c : ℝ f : α →ₛ E hf : Integrable ↑f ⊢ (fun x x_1 => x • x_1) c 0 = 0 ** dsimp only ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T c : ℝ f : α →ₛ E hf : Integrable ↑f ⊢ c • 0 = 0 ** rw [smul_zero] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T c : ℝ f : α →ₛ E hf : Integrable ↑f b : E x✝ : b ∈ SimpleFunc.range f ⊢ ↑(T (↑f ⁻¹' {b})) (c • b) = c • ↑(T (↑f ⁻¹' {b})) b ** rw [ContinuousLinearMap.map_smul (T (f ⁻¹' {b})) c b] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T c : ℝ f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, c • ↑(T (↑f ⁻¹' {x})) x = c • setToSimpleFunc T f ** simp only [setToSimpleFunc, smul_sum, smul_smul, mul_comm] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_smul ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹¹ : NormedAddCommGroup E✝ inst✝¹⁰ : NormedSpace ℝ E✝ inst✝⁹ : NormedAddCommGroup F inst✝⁸ : NormedSpace ℝ F inst✝⁷ : NormedAddCommGroup F' inst✝⁶ : NormedSpace ℝ F' inst✝⁵ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α E : Type u_7 inst✝⁴ : NormedAddCommGroup E inst✝³ : NormedField 𝕜 inst✝² : NormedSpace 𝕜 E inst✝¹ : NormedSpace ℝ E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T (c • f) = ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) (c • x) ** rw [smul_eq_map c f, map_setToSimpleFunc T h_add hf] ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹¹ : NormedAddCommGroup E✝ inst✝¹⁰ : NormedSpace ℝ E✝ inst✝⁹ : NormedAddCommGroup F inst✝⁸ : NormedSpace ℝ F inst✝⁷ : NormedAddCommGroup F' inst✝⁶ : NormedSpace ℝ F' inst✝⁵ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α E : Type u_7 inst✝⁴ : NormedAddCommGroup E inst✝³ : NormedField 𝕜 inst✝² : NormedSpace 𝕜 E inst✝¹ : NormedSpace ℝ E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : α →ₛ E hf : Integrable ↑f ⊢ (fun x x_1 => x • x_1) c 0 = 0 ** dsimp only ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹¹ : NormedAddCommGroup E✝ inst✝¹⁰ : NormedSpace ℝ E✝ inst✝⁹ : NormedAddCommGroup F inst✝⁸ : NormedSpace ℝ F inst✝⁷ : NormedAddCommGroup F' inst✝⁶ : NormedSpace ℝ F' inst✝⁵ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α E : Type u_7 inst✝⁴ : NormedAddCommGroup E inst✝³ : NormedField 𝕜 inst✝² : NormedSpace 𝕜 E inst✝¹ : NormedSpace ℝ E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : α →ₛ E hf : Integrable ↑f ⊢ c • 0 = 0 ** rw [smul_zero] ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹¹ : NormedAddCommGroup E✝ inst✝¹⁰ : NormedSpace ℝ E✝ inst✝⁹ : NormedAddCommGroup F inst✝⁸ : NormedSpace ℝ F inst✝⁷ : NormedAddCommGroup F' inst✝⁶ : NormedSpace ℝ F' inst✝⁵ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α E : Type u_7 inst✝⁴ : NormedAddCommGroup E inst✝³ : NormedField 𝕜 inst✝² : NormedSpace 𝕜 E inst✝¹ : NormedSpace ℝ E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : α →ₛ E hf : Integrable ↑f b : E x✝ : b ∈ SimpleFunc.range f ⊢ ↑(T (↑f ⁻¹' {b})) (c • b) = c • ↑(T (↑f ⁻¹' {b})) b ** rw [h_smul] ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹¹ : NormedAddCommGroup E✝ inst✝¹⁰ : NormedSpace ℝ E✝ inst✝⁹ : NormedAddCommGroup F inst✝⁸ : NormedSpace ℝ F inst✝⁷ : NormedAddCommGroup F' inst✝⁶ : NormedSpace ℝ F' inst✝⁵ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α E : Type u_7 inst✝⁴ : NormedAddCommGroup E inst✝³ : NormedField 𝕜 inst✝² : NormedSpace 𝕜 E inst✝¹ : NormedSpace ℝ E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, c • ↑(T (↑f ⁻¹' {x})) x = c • setToSimpleFunc T f ** simp only [setToSimpleFunc, smul_sum, smul_smul, mul_comm] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_mono_left ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T T' : Set α → F →L[ℝ] G'' hTT' : ∀ (s : Set α) (x : F), ↑(T s) x ≤ ↑(T' s) x f : α →ₛ F ⊢ setToSimpleFunc T f ≤ setToSimpleFunc T' f ** simp_rw [setToSimpleFunc] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T T' : Set α → F →L[ℝ] G'' hTT' : ∀ (s : Set α) (x : F), ↑(T s) x ≤ ↑(T' s) x f : α →ₛ F ⊢ ∑ x in SimpleFunc.range f, ↑(T (↑f ⁻¹' {x})) x ≤ ∑ x in SimpleFunc.range f, ↑(T' (↑f ⁻¹' {x})) x ** exact sum_le_sum fun i _ => hTT' _ i ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_mono_left' ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T T' : Set α → E →L[ℝ] G'' hTT' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : E), ↑(T s) x ≤ ↑(T' s) x f : α →ₛ E hf : Integrable ↑f ⊢ setToSimpleFunc T f ≤ setToSimpleFunc T' f ** refine' sum_le_sum fun i _ => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T T' : Set α → E →L[ℝ] G'' hTT' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : E), ↑(T s) x ≤ ↑(T' s) x f : α →ₛ E hf : Integrable ↑f i : E x✝ : i ∈ SimpleFunc.range f ⊢ ↑(T (↑f ⁻¹' {i})) i ≤ ↑(T' (↑f ⁻¹' {i})) i ** by_cases h0 : i = 0 ** case pos α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T T' : Set α → E →L[ℝ] G'' hTT' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : E), ↑(T s) x ≤ ↑(T' s) x f : α →ₛ E hf : Integrable ↑f i : E x✝ : i ∈ SimpleFunc.range f h0 : i = 0 ⊢ ↑(T (↑f ⁻¹' {i})) i ≤ ↑(T' (↑f ⁻¹' {i})) i ** simp [h0] ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T T' : Set α → E →L[ℝ] G'' hTT' : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : E), ↑(T s) x ≤ ↑(T' s) x f : α →ₛ E hf : Integrable ↑f i : E x✝ : i ∈ SimpleFunc.range f h0 : ¬i = 0 ⊢ ↑(T (↑f ⁻¹' {i})) i ≤ ↑(T' (↑f ⁻¹' {i})) i ** exact hTT' _ (measurableSet_fiber _ _) (measure_preimage_lt_top_of_integrable _ hf h0) i ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_nonneg ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α) (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f ⊢ 0 ≤ setToSimpleFunc T f ** refine' sum_nonneg fun i hi => hT_nonneg _ i _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α) (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f i : G' hi : i ∈ SimpleFunc.range f ⊢ 0 ≤ i ** rw [mem_range] at hi ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α) (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f i : G' hi : i ∈ Set.range ↑f ⊢ 0 ≤ i ** obtain ⟨y, hy⟩ := Set.mem_range.mp hi ** case intro α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α) (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f i : G' hi : i ∈ Set.range ↑f y : α hy : ↑f y = i ⊢ 0 ≤ i ** rw [← hy] ** case intro α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α) (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f i : G' hi : i ∈ Set.range ↑f y : α hy : ↑f y = i ⊢ 0 ≤ ↑f y ** refine' le_trans _ (hf y) ** case intro α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' m : MeasurableSpace α T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α) (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f i : G' hi : i ∈ Set.range ↑f y : α hy : ↑f y = i ⊢ 0 ≤ ↑0 y ** simp ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_nonneg' ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f ⊢ 0 ≤ setToSimpleFunc T f ** refine' sum_nonneg fun i hi => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ SimpleFunc.range f ⊢ 0 ≤ ↑(T (↑f ⁻¹' {i})) i ** by_cases h0 : i = 0 ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ SimpleFunc.range f h0 : ¬i = 0 ⊢ 0 ≤ ↑(T (↑f ⁻¹' {i})) i ** refine'
hT_nonneg _ (measurableSet_fiber _ _) (measure_preimage_lt_top_of_integrable _ hfi h0) i _ ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ SimpleFunc.range f h0 : ¬i = 0 ⊢ 0 ≤ i ** rw [mem_range] at hi ** case neg α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ Set.range ↑f h0 : ¬i = 0 ⊢ 0 ≤ i ** obtain ⟨y, hy⟩ := Set.mem_range.mp hi ** case neg.intro α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ Set.range ↑f h0 : ¬i = 0 y : α hy : ↑f y = i ⊢ 0 ≤ i ** rw [← hy] ** case neg.intro α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ Set.range ↑f h0 : ¬i = 0 y : α hy : ↑f y = i ⊢ 0 ≤ ↑f y ** convert hf y ** case pos α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f : α →ₛ G' hf : 0 ≤ f hfi : Integrable ↑f i : G' hi : i ∈ SimpleFunc.range f h0 : i = 0 ⊢ 0 ≤ ↑(T (↑f ⁻¹' {i})) i ** simp [h0] ** Qed
| |
MeasureTheory.SimpleFunc.setToSimpleFunc_mono ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' h_add : FinMeasAdditive μ T hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f g : α →ₛ G' hfi : Integrable ↑f hgi : Integrable ↑g hfg : f ≤ g ⊢ setToSimpleFunc T f ≤ setToSimpleFunc T g ** rw [← sub_nonneg, ← setToSimpleFunc_sub T h_add hgi hfi] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' h_add : FinMeasAdditive μ T hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f g : α →ₛ G' hfi : Integrable ↑f hgi : Integrable ↑g hfg : f ≤ g ⊢ 0 ≤ setToSimpleFunc T (g - f) ** refine' setToSimpleFunc_nonneg' T hT_nonneg _ _ (hgi.sub hfi) ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' h_add : FinMeasAdditive μ T hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f g : α →ₛ G' hfi : Integrable ↑f hgi : Integrable ↑g hfg : f ≤ g ⊢ 0 ≤ g - f ** intro x ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' h_add : FinMeasAdditive μ T hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f g : α →ₛ G' hfi : Integrable ↑f hgi : Integrable ↑g hfg : f ≤ g x : α ⊢ ↑0 x ≤ ↑(g - f) x ** simp only [coe_sub, sub_nonneg, coe_zero, Pi.zero_apply, Pi.sub_apply] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹⁰ : NormedAddCommGroup E inst✝⁹ : NormedSpace ℝ E inst✝⁸ : NormedAddCommGroup F inst✝⁷ : NormedSpace ℝ F inst✝⁶ : NormedAddCommGroup F' inst✝⁵ : NormedSpace ℝ F' inst✝⁴ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α G' : Type u_7 G'' : Type u_8 inst✝³ : NormedLatticeAddCommGroup G'' inst✝² : NormedSpace ℝ G'' inst✝¹ : NormedLatticeAddCommGroup G' inst✝ : NormedSpace ℝ G' T : Set α → G' →L[ℝ] G'' h_add : FinMeasAdditive μ T hT_nonneg : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ∀ (x : G'), 0 ≤ x → 0 ≤ ↑(T s) x f g : α →ₛ G' hfi : Integrable ↑f hgi : Integrable ↑g hfg : f ≤ g x : α ⊢ ↑f x ≤ ↑g x ** exact hfg x ** Qed
| |
MeasureTheory.SimpleFunc.norm_setToSimpleFunc_le_sum_op_norm ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F' →L[ℝ] F f : α →ₛ F' ⊢ ∑ x in SimpleFunc.range f, ‖↑(T (↑f ⁻¹' {x})) x‖ ≤ ∑ x in SimpleFunc.range f, ‖T (↑f ⁻¹' {x})‖ * ‖x‖ ** refine' Finset.sum_le_sum fun b _ => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m✝ : MeasurableSpace α μ : Measure α m : MeasurableSpace α T : Set α → F' →L[ℝ] F f : α →ₛ F' b : F' x✝ : b ∈ SimpleFunc.range f ⊢ ‖↑(T (↑f ⁻¹' {b})) b‖ ≤ ‖T (↑f ⁻¹' {b})‖ * ‖b‖ ** simp_rw [ContinuousLinearMap.le_op_norm] ** Qed
| |
MeasureTheory.SimpleFunc.norm_setToSimpleFunc_le_sum_mul_norm ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ F ⊢ ∑ x in SimpleFunc.range f, ‖T (↑f ⁻¹' {x})‖ * ‖x‖ ≤ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ** gcongr ** case h.h α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ F i✝ : F a✝ : i✝ ∈ SimpleFunc.range f ⊢ ‖T (↑f ⁻¹' {i✝})‖ ≤ C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {i✝})) ** exact hT_norm _ <| SimpleFunc.measurableSet_fiber _ _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ F ⊢ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ≤ C * ∑ x in SimpleFunc.range f, ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ** simp_rw [mul_sum, ← mul_assoc] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → F →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ F ⊢ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ≤ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ** rfl ** Qed
| |
MeasureTheory.SimpleFunc.norm_setToSimpleFunc_le_sum_mul_norm_of_integrable ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, ‖T (↑f ⁻¹' {x})‖ * ‖x‖ ≤ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ** refine' Finset.sum_le_sum fun b hb => _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f b : E hb : b ∈ SimpleFunc.range f ⊢ ‖T (↑f ⁻¹' {b})‖ * ‖b‖ ≤ C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {b})) * ‖b‖ ** obtain rfl | hb := eq_or_ne b 0 ** case inr α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f b : E hb✝ : b ∈ SimpleFunc.range f hb : b ≠ 0 ⊢ ‖T (↑f ⁻¹' {b})‖ * ‖b‖ ≤ C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {b})) * ‖b‖ ** gcongr ** case inr.h α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f b : E hb✝ : b ∈ SimpleFunc.range f hb : b ≠ 0 ⊢ ‖T (↑f ⁻¹' {b})‖ ≤ C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {b})) ** exact hT_norm _ (SimpleFunc.measurableSet_fiber _ _) <|
SimpleFunc.measure_preimage_lt_top_of_integrable _ hf hb ** case inl α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f hb : 0 ∈ SimpleFunc.range f ⊢ ‖T (↑f ⁻¹' {0})‖ * ‖0‖ ≤ C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {0})) * ‖0‖ ** simp ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ≤ C * ∑ x in SimpleFunc.range f, ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ** simp_rw [mul_sum, ← mul_assoc] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁶ : NormedAddCommGroup E inst✝⁵ : NormedSpace ℝ E inst✝⁴ : NormedAddCommGroup F inst✝³ : NormedSpace ℝ F inst✝² : NormedAddCommGroup F' inst✝¹ : NormedSpace ℝ F' inst✝ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α T : Set α → E →L[ℝ] F' C : ℝ hT_norm : ∀ (s : Set α), MeasurableSet s → ↑↑μ s < ⊤ → ‖T s‖ ≤ C * ENNReal.toReal (↑↑μ s) f : α →ₛ E hf : Integrable ↑f ⊢ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ≤ ∑ x in SimpleFunc.range f, C * ENNReal.toReal (↑↑μ (↑f ⁻¹' {x})) * ‖x‖ ** rfl ** Qed
| |
MeasureTheory.L1.SimpleFunc.setToL1S_congr_measure ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' ⊢ setToL1S T f = setToL1S T f' ** refine' SimpleFunc.setToSimpleFunc_congr T h_zero h_add (SimpleFunc.integrable f) _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' ⊢ ↑(toSimpleFunc f) =ᵐ[μ] ↑(toSimpleFunc f') ** refine' (toSimpleFunc_eq_toFun f).trans _ ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' ⊢ ↑↑↑f =ᵐ[μ] ↑(toSimpleFunc f') ** suffices : (f' : α → E) =ᵐ[μ] simpleFunc.toSimpleFunc f' ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' this : ↑↑↑f' =ᵐ[μ] ↑(toSimpleFunc f') ⊢ ↑↑↑f =ᵐ[μ] ↑(toSimpleFunc f') case this α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' ⊢ ↑↑↑f' =ᵐ[μ] ↑(toSimpleFunc f') ** exact h.trans this ** case this α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' ⊢ ↑↑↑f' =ᵐ[μ] ↑(toSimpleFunc f') ** have goal' : (f' : α → E) =ᵐ[μ'] simpleFunc.toSimpleFunc f' := (toSimpleFunc_eq_toFun f').symm ** case this α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E μ' : Measure α T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T hμ : μ ≪ μ' f : { x // x ∈ simpleFunc E 1 μ } f' : { x // x ∈ simpleFunc E 1 μ' } h : ↑↑↑f =ᵐ[μ] ↑↑↑f' goal' : ↑↑↑f' =ᵐ[μ'] ↑(toSimpleFunc f') ⊢ ↑↑↑f' =ᵐ[μ] ↑(toSimpleFunc f') ** exact hμ.ae_eq goal' ** Qed
| |
MeasureTheory.L1.SimpleFunc.setToL1S_neg ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T f : { x // x ∈ simpleFunc E 1 μ } ⊢ setToL1S T (-f) = -setToL1S T f ** simp_rw [setToL1S] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T f : { x // x ∈ simpleFunc E 1 μ } ⊢ SimpleFunc.setToSimpleFunc T (toSimpleFunc (-f)) = -SimpleFunc.setToSimpleFunc T (toSimpleFunc f) ** have : simpleFunc.toSimpleFunc (-f) =ᵐ[μ] ⇑(-simpleFunc.toSimpleFunc f) :=
neg_toSimpleFunc f ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T f : { x // x ∈ simpleFunc E 1 μ } this : ↑(toSimpleFunc (-f)) =ᵐ[μ] ↑(-toSimpleFunc f) ⊢ SimpleFunc.setToSimpleFunc T (toSimpleFunc (-f)) = -SimpleFunc.setToSimpleFunc T (toSimpleFunc f) ** rw [SimpleFunc.setToSimpleFunc_congr T h_zero h_add (SimpleFunc.integrable _) this] ** α : Type u_1 E : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝⁸ : NormedAddCommGroup E inst✝⁷ : NormedSpace ℝ E inst✝⁶ : NormedAddCommGroup F inst✝⁵ : NormedSpace ℝ F inst✝⁴ : NormedAddCommGroup F' inst✝³ : NormedSpace ℝ F' inst✝² : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝¹ : NormedField 𝕜 inst✝ : NormedSpace 𝕜 E T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T f : { x // x ∈ simpleFunc E 1 μ } this : ↑(toSimpleFunc (-f)) =ᵐ[μ] ↑(-toSimpleFunc f) ⊢ SimpleFunc.setToSimpleFunc T (-toSimpleFunc f) = -SimpleFunc.setToSimpleFunc T (toSimpleFunc f) ** exact SimpleFunc.setToSimpleFunc_neg T h_add (SimpleFunc.integrable f) ** Qed
| |
MeasureTheory.L1.SimpleFunc.setToL1S_smul ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹² : NormedAddCommGroup E✝ inst✝¹¹ : NormedSpace ℝ E✝ inst✝¹⁰ : NormedAddCommGroup F inst✝⁹ : NormedSpace ℝ F inst✝⁸ : NormedAddCommGroup F' inst✝⁷ : NormedSpace ℝ F' inst✝⁶ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝⁵ : NormedField 𝕜 inst✝⁴ : NormedSpace 𝕜 E✝ E : Type u_7 inst✝³ : NormedAddCommGroup E inst✝² : NormedSpace ℝ E inst✝¹ : NormedSpace 𝕜 E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : { x // x ∈ simpleFunc E 1 μ } ⊢ setToL1S T (c • f) = c • setToL1S T f ** simp_rw [setToL1S] ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹² : NormedAddCommGroup E✝ inst✝¹¹ : NormedSpace ℝ E✝ inst✝¹⁰ : NormedAddCommGroup F inst✝⁹ : NormedSpace ℝ F inst✝⁸ : NormedAddCommGroup F' inst✝⁷ : NormedSpace ℝ F' inst✝⁶ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝⁵ : NormedField 𝕜 inst✝⁴ : NormedSpace 𝕜 E✝ E : Type u_7 inst✝³ : NormedAddCommGroup E inst✝² : NormedSpace ℝ E inst✝¹ : NormedSpace 𝕜 E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : { x // x ∈ simpleFunc E 1 μ } ⊢ SimpleFunc.setToSimpleFunc T (toSimpleFunc (c • f)) = c • SimpleFunc.setToSimpleFunc T (toSimpleFunc f) ** rw [← SimpleFunc.setToSimpleFunc_smul T h_add h_smul c (SimpleFunc.integrable f)] ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹² : NormedAddCommGroup E✝ inst✝¹¹ : NormedSpace ℝ E✝ inst✝¹⁰ : NormedAddCommGroup F inst✝⁹ : NormedSpace ℝ F inst✝⁸ : NormedAddCommGroup F' inst✝⁷ : NormedSpace ℝ F' inst✝⁶ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝⁵ : NormedField 𝕜 inst✝⁴ : NormedSpace 𝕜 E✝ E : Type u_7 inst✝³ : NormedAddCommGroup E inst✝² : NormedSpace ℝ E inst✝¹ : NormedSpace 𝕜 E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : { x // x ∈ simpleFunc E 1 μ } ⊢ SimpleFunc.setToSimpleFunc T (toSimpleFunc (c • f)) = SimpleFunc.setToSimpleFunc T (c • toSimpleFunc f) ** refine' SimpleFunc.setToSimpleFunc_congr T h_zero h_add (SimpleFunc.integrable _) _ ** α : Type u_1 E✝ : Type u_2 F : Type u_3 F' : Type u_4 G : Type u_5 𝕜 : Type u_6 p : ℝ≥0∞ inst✝¹² : NormedAddCommGroup E✝ inst✝¹¹ : NormedSpace ℝ E✝ inst✝¹⁰ : NormedAddCommGroup F inst✝⁹ : NormedSpace ℝ F inst✝⁸ : NormedAddCommGroup F' inst✝⁷ : NormedSpace ℝ F' inst✝⁶ : NormedAddCommGroup G m : MeasurableSpace α μ : Measure α inst✝⁵ : NormedField 𝕜 inst✝⁴ : NormedSpace 𝕜 E✝ E : Type u_7 inst✝³ : NormedAddCommGroup E inst✝² : NormedSpace ℝ E inst✝¹ : NormedSpace 𝕜 E inst✝ : NormedSpace 𝕜 F T : Set α → E →L[ℝ] F h_zero : ∀ (s : Set α), MeasurableSet s → ↑↑μ s = 0 → T s = 0 h_add : FinMeasAdditive μ T h_smul : ∀ (c : 𝕜) (s : Set α) (x : E), ↑(T s) (c • x) = c • ↑(T s) x c : 𝕜 f : { x // x ∈ simpleFunc E 1 μ } ⊢ ↑(toSimpleFunc (c • f)) =ᵐ[μ] ↑(c • toSimpleFunc f) ** exact smul_toSimpleFunc c f ** Qed
|
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.