Skip to content

Commit

Permalink
feat(analysis/normed_space/normed_group_hom): add norm_noninc.neg (#9658
Browse files Browse the repository at this point in the history
)

From LTE.
  • Loading branch information
riccardobrasca committed Oct 11, 2021
1 parent df132fe commit c2a30be
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/analysis/normed_space/normed_group_hom.lean
Expand Up @@ -548,6 +548,9 @@ lemma comp {g : normed_group_hom V₂ V₃} {f : normed_group_hom V₁ V₂}
(g.comp f).norm_noninc :=
λ v, (hg (f v)).trans (hf v)

@[simp] lemma neg_iff {f : normed_group_hom V₁ V₂} : (-f).norm_noninc ↔ f.norm_noninc :=
⟨λ h x, by { simpa using h x }, λ h x, (norm_neg (f x)).le.trans (h x)⟩

end norm_noninc

section isometry
Expand Down

0 comments on commit c2a30be

Please sign in to comment.