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

Commit c2a30be

Browse files
feat(analysis/normed_space/normed_group_hom): add norm_noninc.neg (#9658)
From LTE.
1 parent df132fe commit c2a30be

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/analysis/normed_space/normed_group_hom.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -548,6 +548,9 @@ lemma comp {g : normed_group_hom V₂ V₃} {f : normed_group_hom V₁ V₂}
548548
(g.comp f).norm_noninc :=
549549
λ v, (hg (f v)).trans (hf v)
550550

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

553556
section isometry

0 commit comments

Comments
 (0)