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

Commit def4814

Browse files
dupuisfhrmacbeth
andcommitted
refactor(topology/algebra/module): continuous semilinear maps (#9539)
Generalize the theory of continuous linear maps to the semilinear setting. We introduce a notation `∘L` for composition of continuous linear (i.e., not semilinear) maps, used sporadically to help with unification. See #8857 for a discussion of a related problem and fix. Co-authored-by: Frédéric Dupuis <dupuisf@iro.umontreal.ca> Co-authored-by: Heather Macbeth <25316162+hrmacbeth@users.noreply.github.com>
1 parent fefd8a3 commit def4814

File tree

3 files changed

+392
-279
lines changed

3 files changed

+392
-279
lines changed

src/analysis/complex/conformal.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -74,7 +74,7 @@ variables {f : ℂ → ℂ} {z : ℂ} {g : ℂ →L[ℝ] ℂ}
7474

7575
lemma is_conformal_map.is_complex_or_conj_linear (h : is_conformal_map g) :
7676
(∃ (map : ℂ →L[ℂ] ℂ), map.restrict_scalars ℝ = g) ∨
77-
(∃ (map : ℂ →L[ℂ] ℂ), map.restrict_scalars ℝ = g.comp ↑conj_cle) :=
77+
(∃ (map : ℂ →L[ℂ] ℂ), map.restrict_scalars ℝ = g ∘L ↑conj_cle) :=
7878
begin
7979
rcases h with ⟨c, hc, li, hg⟩,
8080
rcases linear_isometry_complex (li.to_linear_isometry_equiv rfl) with ⟨a, ha⟩,
@@ -100,15 +100,15 @@ end
100100
lemma is_conformal_map_iff_is_complex_or_conj_linear:
101101
is_conformal_map g ↔
102102
((∃ (map : ℂ →L[ℂ] ℂ), map.restrict_scalars ℝ = g) ∨
103-
(∃ (map : ℂ →L[ℂ] ℂ), map.restrict_scalars ℝ = g.comp ↑conj_cle)) ∧ g ≠ 0 :=
103+
(∃ (map : ℂ →L[ℂ] ℂ), map.restrict_scalars ℝ = g ∘L ↑conj_cle)) ∧ g ≠ 0 :=
104104
begin
105105
split,
106106
{ exact λ h, ⟨h.is_complex_or_conj_linear, h.ne_zero⟩, },
107107
{ rintros ⟨⟨map, rfl⟩ | ⟨map, hmap⟩, h₂⟩,
108108
{ refine is_conformal_map_complex_linear _,
109109
contrapose! h₂ with w,
110110
simp [w] },
111-
{ have minor₁ : g = (map.restrict_scalars ℝ).comp ↑conj_cle,
111+
{ have minor₁ : g = (map.restrict_scalars ℝ) ∘L ↑conj_cle,
112112
{ ext1,
113113
simp [hmap] },
114114
rw minor₁ at ⊢ h₂,

src/analysis/normed_space/complemented.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -91,7 +91,7 @@ end
9191
def linear_proj_of_closed_compl (h : is_compl p q) (hp : is_closed (p : set E))
9292
(hq : is_closed (q : set E)) :
9393
E →L[𝕜] p :=
94-
(continuous_linear_map.fst 𝕜 p q).comp $ (prod_equiv_of_closed_compl p q h hp hq).symm
94+
(continuous_linear_map.fst 𝕜 p q) ∘L ↑(prod_equiv_of_closed_compl p q h hp hq).symm
9595

9696
variables {p q}
9797

0 commit comments

Comments
 (0)