Skip to content

Commit

Permalink
feat(measure_theory/measure/vector_measure): add `mutually_singular.n…
Browse files Browse the repository at this point in the history
…eg` (#9282)
  • Loading branch information
JasonKYi committed Sep 21, 2021
1 parent 78340e3 commit 4cee743
Showing 1 changed file with 25 additions and 0 deletions.
25 changes: 25 additions & 0 deletions src/measure_theory/measure/vector_measure.lean
Expand Up @@ -1088,6 +1088,31 @@ lemma smul_left {R : Type*} [semiring R] [distrib_mul_action R M] [topological_s
[has_continuous_smul R M] (r : R) (h : v ⊥ᵥ w) : r • v ⊥ᵥ w :=
(smul_right r h.symm).symm

lemma neg_left {M : Type*} [add_comm_group M] [topological_space M] [topological_add_group M]
{v : vector_measure α M} {w : vector_measure α N} (h : v ⊥ᵥ w) : -v ⊥ᵥ w :=
begin
obtain ⟨u, hmu, hu₁, hu₂⟩ := h,
refine ⟨u, hmu, λ s hs, _, hu₂⟩,
rw [neg_apply v s, neg_eq_zero],
exact hu₁ s hs
end

lemma neg_right {N : Type*} [add_comm_group N] [topological_space N] [topological_add_group N]
{v : vector_measure α M} {w : vector_measure α N} (h : v ⊥ᵥ w) : v ⊥ᵥ -w :=
h.symm.neg_left.symm

@[simp]
lemma neg_left_iff {M : Type*} [add_comm_group M] [topological_space M] [topological_add_group M]
{v : vector_measure α M} {w : vector_measure α N} :
-v ⊥ᵥ w ↔ v ⊥ᵥ w :=
⟨λ h, neg_neg v ▸ h.neg_left, neg_left⟩

@[simp]
lemma neg_right_iff {N : Type*} [add_comm_group N] [topological_space N] [topological_add_group N]
{v : vector_measure α M} {w : vector_measure α N} :
v ⊥ᵥ -w ↔ v ⊥ᵥ w :=
⟨λ h, neg_neg w ▸ h.neg_right, neg_right⟩

end mutually_singular

section trim
Expand Down

0 comments on commit 4cee743

Please sign in to comment.