Skip to content

Commit

Permalink
chore(linear_algebra/affine_space/basic): split (#4767)
Browse files Browse the repository at this point in the history
* Split `linear_algebra/affine_space/basic` into two files: `affine_map` and `affine_subspace`.
* Move notation `affine_space` to the bottom of `algebra/add_torsor`.
  • Loading branch information
urkud committed Oct 28, 2020
1 parent 4d1da54 commit 7807f3d
Show file tree
Hide file tree
Showing 12 changed files with 1,581 additions and 1,535 deletions.
19 changes: 11 additions & 8 deletions src/algebra/add_torsor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -23,14 +23,17 @@ defines the notation `+ᵥ` for adding a group element to a point and
## Implementation notes
Affine spaces are the motivating example of torsors of additive group
actions. It may be appropriate to refactor in terms of the general
definition of group actions, via `to_additive`, when there is a use
for multiplicative torsors (currently mathlib only develops the theory
of group actions for multiplicative group actions). The variable `G`
is an explicit rather than implicit argument to lemmas because
otherwise the elaborator sometimes has problems inferring appropriate
types and type class instances.
Affine spaces are the motivating example of torsors of additive group actions. It may be appropriate
to refactor in terms of the general definition of group actions, via `to_additive`, when there is a
use for multiplicative torsors (currently mathlib only develops the theory of group actions for
multiplicative group actions).
## Notations
* `v +ᵥ p` is a notation for `has_vadd.vadd`, the left action of an additive monoid;
* `p₁ -ᵥ p₂` is a notation for `has_vsub.vsub`, difference between two points in an additive torsor
as an element of the corresponding additive group;
## References
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/convex/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Alexander Bentkamp, Yury Kudriashov
import data.set.intervals.ord_connected
import data.set.intervals.image_preimage
import data.complex.module
import linear_algebra.affine_space.basic
import linear_algebra.affine_space.affine_map
import algebra.module.ordered


Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/mazur_ulam.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Author: Yury Kudryashov
import analysis.normed_space.point_reflection
import topology.instances.real_vector_space
import analysis.normed_space.add_torsor
import linear_algebra.affine_space.basic
import linear_algebra.affine_space.affine_map

/-!
# Mazur-Ulam Theorem
Expand Down
3 changes: 2 additions & 1 deletion src/linear_algebra/affine_space/affine_equiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Yury G. Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: Yury G. Kudryashov
-/
import linear_algebra.affine_space.basic
import linear_algebra.affine_space.affine_map

/-!
# Affine equivalences
Expand All @@ -28,6 +28,7 @@ affine space, affine equivalence
-/

open function set
open_locale affine

/-- An affine equivalence is an equivalence between affine spaces such that both forward
and inverse maps are affine.
Expand Down
Loading

0 comments on commit 7807f3d

Please sign in to comment.