Skip to content

Commit

Permalink
feat(analysis/normed/group/SemiNormedGroup): add iso_isometry_of_norm…
Browse files Browse the repository at this point in the history
…_noninc (#9710)

From LTE.
  • Loading branch information
riccardobrasca committed Oct 16, 2021
1 parent 5ac586a commit 3d99926
Showing 1 changed file with 11 additions and 0 deletions.
11 changes: 11 additions & 0 deletions src/analysis/normed/group/SemiNormedGroup.lean
Expand Up @@ -55,6 +55,17 @@ instance has_zero_object : limits.has_zero_object SemiNormedGroup.{u} :=
{ default := 0,
uniq := λ f, by ext } }

lemma iso_isometry_of_norm_noninc {V W : SemiNormedGroup} (i : V ≅ W)
(h1 : i.hom.norm_noninc) (h2 : i.inv.norm_noninc) :
isometry i.hom :=
begin
apply normed_group_hom.isometry_of_norm,
intro v,
apply le_antisymm (h1 v),
calc ∥v∥ = ∥i.inv (i.hom v)∥ : by rw [coe_hom_inv_id]
... ≤ ∥i.hom v∥ : h2 _,
end

end SemiNormedGroup

/--
Expand Down

0 comments on commit 3d99926

Please sign in to comment.