File tree Expand file tree Collapse file tree 2 files changed +43
-0
lines changed
Mathlib/Analysis/Calculus Expand file tree Collapse file tree 2 files changed +43
-0
lines changed Original file line number Diff line number Diff line change @@ -455,6 +455,7 @@ import Mathlib.Analysis.BoxIntegral.Partition.Measure
455
455
import Mathlib.Analysis.BoxIntegral.Partition.Split
456
456
import Mathlib.Analysis.BoxIntegral.Partition.SubboxInduction
457
457
import Mathlib.Analysis.BoxIntegral.Partition.Tagged
458
+ import Mathlib.Analysis.Calculus.AffineMap
458
459
import Mathlib.Analysis.Calculus.BumpFunctionInner
459
460
import Mathlib.Analysis.Calculus.Conformal.InnerProduct
460
461
import Mathlib.Analysis.Calculus.Conformal.NormedSpace
Original file line number Diff line number Diff line change
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
You canβt perform that action at this time.
0 commit comments