Skip to content

Commit f35b744

Browse files
authored
Merge pull request #272 from teorth:fix
fix gap in 3.1
2 parents 85e4153 + bd1add2 commit f35b744

File tree

2 files changed

+3
-4
lines changed

2 files changed

+3
-4
lines changed

analysis/Analysis/Section_11_4.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -30,8 +30,7 @@ theorem IntegrableOn.smul {I: BoundedInterval} (c:ℝ) {f:ℝ → ℝ} (hf: Inte
3030
sorry
3131

3232
theorem IntegrableOn.neg {I: BoundedInterval} {f:ℝ → ℝ} (hf: IntegrableOn f I) :
33-
IntegrableOn (-f) I ∧ integ (-f) I = -integ f I := by
34-
have := IntegrableOn.smul (-1) hf; simp_all; tauto
33+
IntegrableOn (-f) I ∧ integ (-f) I = -integ f I := by have := IntegrableOn.smul (-1) hf; aesop
3534

3635
/-- Theorem 11.4.1(c) / Exercise 11.4.1 -/
3736
theorem IntegrableOn.sub {I: BoundedInterval} {f g:ℝ → ℝ} (hf: IntegrableOn f I) (hg: IntegrableOn g I) :
@@ -189,7 +188,7 @@ theorem integ_of_mul_nonneg {I: BoundedInterval} {f g:ℝ → ℝ} (hf: Integrab
189188
. peel hf_nonneg with x hx _; specialize hf'min _ hx; aesop
190189
. exact hf'const.max hzero
191190
. apply lt_of_lt_of_le hf'int (hf'const.integ_mono _ (hf'const.max hzero)); simp
192-
intro _ _; simp
191+
intro _; simp
193192
obtain ⟨ f', hf'min, hf'const, hf'int, hf'_nonneg ⟩ := this
194193
have : ∃ g', MinorizesOn g' g I ∧ PiecewiseConstantOn g' I ∧ integ g I - ε < PiecewiseConstantOn.integ g' I ∧ MajorizesOn g' 0 I := by
195194
obtain ⟨ g', hg'min, hg'const, hg'int ⟩ := gt_of_lt_lower_integral hg.1 (show integ g I - ε < lower_integral g I by linarith)

analysis/Analysis/Section_3_1.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -534,7 +534,7 @@ instance SetTheory.Set.instDistribLattice : DistribLattice Set where
534534
le_inf := by sorry
535535
le_sup_inf := by
536536
intro X Y Z; change (X ∪ Y) ∩ (X ∪ Z) ⊆ X ∪ (Y ∩ Z)
537-
rw [←union_inter_distrib_left]; exact subset_self _
537+
rw [←union_inter_distrib_left]
538538

539539
/-- Sets have a minimal element. -/
540540
instance SetTheory.Set.instOrderBot : OrderBot Set where

0 commit comments

Comments
 (0)