Skip to content

Commit

Permalink
Mention notation in docstrings
Browse files Browse the repository at this point in the history
  • Loading branch information
bustercopley committed Mar 1, 2024
1 parent 14b2f1f commit 79fa8b9
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 3 deletions.
4 changes: 2 additions & 2 deletions Mathlib/LinearAlgebra/Alternating/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -64,8 +64,8 @@ section

variable (R M N ι)

/-- An alternating map is a multilinear map that vanishes when two of its arguments are equal.
-/
/-- An alternating map from `ι → M` to `N`, denoted `M [⋀^ι]→ₗ[R] N`,
is a multilinear map that vanishes when two of its arguments are equal. -/
structure AlternatingMap extends MultilinearMap R (fun _ : ι => M) N where
/-- The map is alternating: if `v` has two equal coordinates, then `f v = 0`. -/
map_eq_zero_of_eq' : ∀ (v : ι → M) (i j : ι), v i = v j → i ≠ j → toFun v = 0
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Topology/Algebra/Module/Alternating/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,8 @@ open Function Matrix

open scoped BigOperators

/-- A continuous alternating map is a continuous map from `ι → M` to `N` that is
/-- A continuous alternating map from `ι → M` to `N`, denoted `M [⋀^ι]→L[R] N`,
is a continuous map that is
- multilinear : `f (update m i (c • x)) = c • f (update m i x)` and
`f (update m i (x + y)) = f (update m i x) + f (update m i y)`;
Expand Down

0 comments on commit 79fa8b9

Please sign in to comment.