Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 665cc13

Browse files
committed
chore(topology/algebra/group): review (#4570)
* Ensure that we don't use `[topological_group G]` when it suffices to ask for, e.g., `[has_continuous_mul G]`. * Introduce `[has_continuous_sub]`, add an instance for `nnreal`.
1 parent 952a407 commit 665cc13

File tree

4 files changed

+177
-127
lines changed

4 files changed

+177
-127
lines changed

src/analysis/convex/topology.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -84,11 +84,11 @@ convex_iff_pointwise_add_subset.mpr $ λ a b ha hb hab,
8484
or.elim (classical.em (a = 0))
8585
(λ heq,
8686
have hne : b ≠ 0, by { rw [heq, zero_add] at hab, rw hab, exact one_ne_zero },
87-
by { rw ← image_smul, apply is_open_add_left,
88-
exact is_open_map_smul_of_ne_zero hne _ is_open_interior } )
87+
by { rw ← image_smul,
88+
exact (is_open_map_smul_of_ne_zero hne _ is_open_interior).add_left } )
8989
(λ hne,
90-
by { rw ← image_smul, apply is_open_add_right,
91-
exact is_open_map_smul_of_ne_zero hne _ is_open_interior }),
90+
by { rw ← image_smul,
91+
exact (is_open_map_smul_of_ne_zero hne _ is_open_interior).add_right }),
9292
(subset_interior_iff_subset_of_open h).mpr $ subset.trans
9393
(by { simp only [← image_smul], apply add_subset_add; exact image_subset _ interior_subset })
9494
(convex_iff_pointwise_add_subset.mp hs ha hb hab)

src/measure_theory/borel_space.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -794,7 +794,7 @@ variable [measurable_space α]
794794

795795
lemma measurable.sub_nnreal {f g : α → ℝ≥0} :
796796
measurable f → measurable g → measurable (λ a, f a - g a) :=
797-
nnreal.continuous_sub.measurable2
797+
continuous_sub.measurable2
798798

799799
lemma measurable.nnreal_of_real {f : α → ℝ} (hf : measurable f) :
800800
measurable (λ x, nnreal.of_real (f x)) :=
@@ -876,7 +876,7 @@ end
876876

877877
lemma measurable_sub : measurable (λ p : ennreal × ennreal, p.1 - p.2) :=
878878
by apply measurable_of_measurable_nnreal_nnreal;
879-
simp [← ennreal.coe_sub, nnreal.continuous_sub.measurable.ennreal_coe]
879+
simp [← ennreal.coe_sub, continuous_sub.measurable.ennreal_coe]
880880

881881
end ennreal
882882

0 commit comments

Comments
 (0)