Skip to content

Commit

Permalink
feat: gcongr lemmas for Additive/Multiplicative (#18959)
Browse files Browse the repository at this point in the history
From FLT

Co-authored-by: Javier Lopez-Contreras <[email protected]>
  • Loading branch information
YaelDillies and Javier Lopez-Contreras committed Dec 2, 2024
1 parent 7cf8077 commit 1e85f24
Show file tree
Hide file tree
Showing 2 changed files with 11 additions and 1 deletion.
10 changes: 10 additions & 0 deletions Mathlib/Algebra/Order/Monoid/Unbundled/TypeTags.lean
Original file line number Diff line number Diff line change
Expand Up @@ -86,6 +86,11 @@ theorem toMul_le {a b : Additive α} : a.toMul ≤ b.toMul ↔ a ≤ b :=
theorem toMul_lt {a b : Additive α} : a.toMul < b.toMul ↔ a < b :=
Iff.rfl

@[gcongr] alias ⟨_, toMul_mono⟩ := toMul_le
@[gcongr] alias ⟨_, ofMul_mono⟩ := ofMul_le
@[gcongr] alias ⟨_, toMul_strictMono⟩ := toMul_lt
@[gcongr] alias ⟨_, foMul_strictMono⟩ := ofMul_lt

end Additive

namespace Multiplicative
Expand All @@ -108,4 +113,9 @@ theorem toAdd_le {a b : Multiplicative α} : a.toAdd ≤ b.toAdd ↔ a ≤ b :=
theorem toAdd_lt {a b : Multiplicative α} : a.toAdd < b.toAdd ↔ a < b :=
Iff.rfl

@[gcongr] alias ⟨_, toAdd_mono⟩ := toAdd_le
@[gcongr] alias ⟨_, ofAdd_mono⟩ := ofAdd_le
@[gcongr] alias ⟨_, toAdd_strictMono⟩ := toAdd_lt
@[gcongr] alias ⟨_, ofAdd_strictMono⟩ := ofAdd_lt

end Multiplicative
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/OuterMeasure/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -61,7 +61,7 @@ theorem measure_iUnion_le [Countable ι] (s : ι → Set α) : μ (⋃ i, s i)
μ (⋃ i, t i) = μ (⋃ i, disjointed t i) := by rw [iUnion_disjointed]
_ ≤ ∑' i, μ (disjointed t i) :=
OuterMeasureClass.measure_iUnion_nat_le _ _ (disjoint_disjointed _)
_ ≤ ∑' i, μ (t i) := by gcongr; apply disjointed_subset
_ ≤ ∑' i, μ (t i) := by gcongr; exact disjointed_subset ..

theorem measure_biUnion_le {I : Set ι} (μ : F) (hI : I.Countable) (s : ι → Set α) :
μ (⋃ i ∈ I, s i) ≤ ∑' i : I, μ (s i) := by
Expand Down

0 comments on commit 1e85f24

Please sign in to comment.