Skip to content

Commit

Permalink
chore(analysis/normed_space/multilinear): use notation (#13452)
Browse files Browse the repository at this point in the history
* use notation `A [×n]→L[𝕜] B`;
* use `A → B` instead of `Π x : A, B`.
  • Loading branch information
urkud committed Apr 15, 2022
1 parent d81cedb commit 6a5764b
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/analysis/normed_space/multilinear.lean
Expand Up @@ -660,8 +660,8 @@ namespace continuous_multilinear_map
these variables, and fixing the other ones equal to a given value `z`. It is denoted by
`f.restr s hk z`, where `hk` is a proof that the cardinality of `s` is `k`. The implicit
identification between `fin k` and `s` that we use is the canonical (increasing) bijection. -/
def restr {k n : ℕ} (f : (G [×n]→L[𝕜] G' : _))
(s : finset (fin n)) (hk : s.card = k) (z : G) : G [×k]→L[𝕜] G' :=
def restr {k n : ℕ} (f : (G [×n]→L[𝕜] G' : _)) (s : finset (fin n)) (hk : s.card = k) (z : G) :
G [×k]→L[𝕜] G' :=
(f.to_multilinear_map.restr s hk z).mk_continuous
(∥f∥ * ∥z∥^(n-k)) $ λ v, multilinear_map.restr_norm_le _ _ _ _ f.le_op_norm _

Expand Down Expand Up @@ -1189,11 +1189,11 @@ variables {n 𝕜 G Ei G'}
(continuous_multilinear_curry_right_equiv 𝕜 Ei G).symm f v x = f (snoc v x) := rfl

@[simp] lemma continuous_multilinear_curry_right_equiv_apply'
(f : G [×n]→L[𝕜] (G →L[𝕜] G')) (v : Π (i : fin n.succ), G) :
(f : G [×n]→L[𝕜] (G →L[𝕜] G')) (v : fin (n + 1) → G) :
continuous_multilinear_curry_right_equiv' 𝕜 n G G' f v = f (init v) (v (last n)) := rfl

@[simp] lemma continuous_multilinear_curry_right_equiv_symm_apply'
(f : G [×n.succ]→L[𝕜] G') (v : Π (i : fin n), G) (x : G) :
(f : G [×n.succ]→L[𝕜] G') (v : fin n G) (x : G) :
(continuous_multilinear_curry_right_equiv' 𝕜 n G G').symm f v x = f (snoc v x) := rfl

@[simp] lemma continuous_multilinear_map.curry_right_norm
Expand Down

0 comments on commit 6a5764b

Please sign in to comment.