Skip to content

Commit

Permalink
feat(analysis/normed_space/basic): norm_entry_le_entrywise_sup_norm (
Browse files Browse the repository at this point in the history
…#12159)

The entries of a matrix are at most the entrywise sup norm.


Co-authored-by: Hans Parshall <hparshall@users.noreply.github.com>
  • Loading branch information
hparshall and hparshall committed Feb 21, 2022
1 parent 1cfbcc6 commit 9a17b55
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions src/analysis/normed_space/basic.lean
Expand Up @@ -791,6 +791,11 @@ def matrix.normed_space {α : Type*} [normed_field α] {n m : Type*} [fintype n]
normed_space α (matrix n m α) :=
pi.normed_space

lemma matrix.norm_entry_le_entrywise_sup_norm {α : Type*} [normed_field α] {n m : Type*} [fintype n]
[fintype m] (M : (matrix n m α)) {i : n} {j : m} :
∥M i j∥ ≤ ∥M∥ :=
(norm_le_pi_norm (M i) j).trans (norm_le_pi_norm M i)

end

end normed_group
Expand Down

0 comments on commit 9a17b55

Please sign in to comment.