Datasets:

Modalities:
Text
Languages:
English
Libraries:
Datasets
License:
Zhangir Azerbayev
squashed?
4365a98
raw
history blame
913 Bytes
/-
Copyright (c) 2021 Oliver Nash. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Oliver Nash
-/
import analysis.normed_space.continuous_affine_map
import analysis.calculus.cont_diff
/-!
# Smooth affine maps
This file contains results about smoothness of affine maps.
## Main definitions:
* `continuous_affine_map.cont_diff`: a continuous affine map is smooth
-/
namespace continuous_affine_map
variables {π•œ V W : Type*} [nontrivially_normed_field π•œ]
variables [normed_add_comm_group V] [normed_space π•œ V]
variables [normed_add_comm_group W] [normed_space π•œ W]
/-- A continuous affine map between normed vector spaces is smooth. -/
lemma cont_diff {n : with_top β„•} (f : V β†’A[π•œ] W) :
cont_diff π•œ n f :=
begin
rw f.decomp,
apply f.cont_linear.cont_diff.add,
simp only,
exact cont_diff_const,
end
end continuous_affine_map