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

Commit d0507e7

Browse files
committed
feat(analysis/normed_space/affine_isometry): subtypeₐᵢ (#16573)
Now that we have `affine_subspace.subtype`, add the corresponding definition as a bundled affine isometry (so resolving a comment about that being missing). The name uses subscript `ₐᵢ` rather than superscript `ᵃⁱ` as in the notation for `affine_isometry` because Lean does not accept the superscript in identifiers.
1 parent f89fa08 commit d0507e7

File tree

1 file changed

+25
-3
lines changed

1 file changed

+25
-3
lines changed

src/analysis/normed_space/affine_isometry.lean

Lines changed: 25 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -197,9 +197,31 @@ instance : monoid (P →ᵃⁱ[𝕜] P) :=
197197

198198
end affine_isometry
199199

200-
-- remark: by analogy with the `linear_isometry` file from which this is adapted, there should
201-
-- follow here a section defining an "inclusion" affine isometry from `p : affine_subspace 𝕜 P`
202-
-- into `P`; we omit this for now
200+
namespace affine_subspace
201+
202+
include V
203+
204+
/-- `affine_subspace.subtype` as an `affine_isometry`. -/
205+
def subtypeₐᵢ (s : affine_subspace 𝕜 P) [nonempty s] : s →ᵃⁱ[𝕜] P :=
206+
{ norm_map := s.direction.subtypeₗᵢ.norm_map,
207+
.. s.subtype }
208+
209+
lemma subtypeₐᵢ_linear (s : affine_subspace 𝕜 P) [nonempty s] :
210+
s.subtypeₐᵢ.linear = s.direction.subtype :=
211+
rfl
212+
213+
@[simp] lemma subtypeₐᵢ_linear_isometry (s : affine_subspace 𝕜 P) [nonempty s] :
214+
s.subtypeₐᵢ.linear_isometry = s.direction.subtypeₗᵢ :=
215+
rfl
216+
217+
@[simp] lemma coe_subtypeₐᵢ (s : affine_subspace 𝕜 P) [nonempty s] : ⇑s.subtypeₐᵢ = s.subtype :=
218+
rfl
219+
220+
@[simp] lemma subtypeₐᵢ_to_affine_map (s : affine_subspace 𝕜 P) [nonempty s] :
221+
s.subtypeₐᵢ.to_affine_map = s.subtype :=
222+
rfl
223+
224+
end affine_subspace
203225

204226
variables (𝕜 P P₂)
205227
include V V₂

0 commit comments

Comments
 (0)