Datasets:
Tasks:
Text Generation
Modalities:
Text
Sub-tasks:
language-modeling
Languages:
English
Size:
100K - 1M
License:
/- | |
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 | |