Skip to content

Commit 1cad7fe

Browse files
committed
feat: port Analysis.Calculus.AffineMap (#4893)
1 parent 697b395 commit 1cad7fe

File tree

2 files changed

+43
-0
lines changed

2 files changed

+43
-0
lines changed

β€ŽMathlib.leanβ€Ž

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -455,6 +455,7 @@ import Mathlib.Analysis.BoxIntegral.Partition.Measure
455455
import Mathlib.Analysis.BoxIntegral.Partition.Split
456456
import Mathlib.Analysis.BoxIntegral.Partition.SubboxInduction
457457
import Mathlib.Analysis.BoxIntegral.Partition.Tagged
458+
import Mathlib.Analysis.Calculus.AffineMap
458459
import Mathlib.Analysis.Calculus.BumpFunctionInner
459460
import Mathlib.Analysis.Calculus.Conformal.InnerProduct
460461
import Mathlib.Analysis.Calculus.Conformal.NormedSpace
Lines changed: 42 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,42 @@
1+
/-
2+
Copyright (c) 2021 Oliver Nash. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Oliver Nash
5+
6+
! This file was ported from Lean 3 source module analysis.calculus.affine_map
7+
! leanprover-community/mathlib commit 839b92fedff9981cf3fe1c1f623e04b0d127f57c
8+
! Please do not edit these lines, except to modify the commit id
9+
! if you have ported upstream changes.
10+
-/
11+
import Mathlib.Analysis.NormedSpace.ContinuousAffineMap
12+
import Mathlib.Analysis.Calculus.ContDiff
13+
14+
/-!
15+
# Smooth affine maps
16+
17+
This file contains results about smoothness of affine maps.
18+
19+
## Main definitions:
20+
21+
* `ContinuousAffineMap.contDiff`: a continuous affine map is smooth
22+
23+
-/
24+
25+
26+
namespace ContinuousAffineMap
27+
28+
variable {π•œ V W : Type _} [NontriviallyNormedField π•œ]
29+
30+
variable [NormedAddCommGroup V] [NormedSpace π•œ V]
31+
32+
variable [NormedAddCommGroup W] [NormedSpace π•œ W]
33+
34+
/-- A continuous affine map between normed vector spaces is smooth. -/
35+
theorem contDiff {n : β„•βˆž} (f : V β†’A[π•œ] W) : ContDiff π•œ n f := by
36+
rw [f.decomp]
37+
apply f.contLinear.contDiff.add
38+
simp only
39+
exact contDiff_const
40+
#align continuous_affine_map.cont_diff ContinuousAffineMap.contDiff
41+
42+
end ContinuousAffineMap

0 commit comments

Comments
Β (0)