Skip to content

Commit

Permalink
feat: define continuous alternating maps (#5678)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Jul 6, 2023
1 parent 0c08a8f commit a691787
Show file tree
Hide file tree
Showing 3 changed files with 623 additions and 1 deletion.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -3031,6 +3031,7 @@ import Mathlib.Topology.Algebra.InfiniteSum.Order
import Mathlib.Topology.Algebra.InfiniteSum.Real
import Mathlib.Topology.Algebra.InfiniteSum.Ring
import Mathlib.Topology.Algebra.Localization
import Mathlib.Topology.Algebra.Module.Alternating
import Mathlib.Topology.Algebra.Module.Basic
import Mathlib.Topology.Algebra.Module.CharacterSpace
import Mathlib.Topology.Algebra.Module.Determinant
Expand Down
8 changes: 7 additions & 1 deletion Mathlib/LinearAlgebra/Alternating.lean
Expand Up @@ -74,7 +74,8 @@ variable (R M N ι)
/-- An alternating map is a multilinear map that vanishes when two of its arguments are equal.
-/
structure AlternatingMap extends MultilinearMap R (fun _ : ι => M) N where
map_eq_zero_of_eq' : ∀ (v : ι → M) (i j : ι) (_ : v i = v j) (_ : i ≠ j), toFun v = 0
/-- 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
#align alternating_map AlternatingMap

end
Expand Down Expand Up @@ -358,6 +359,11 @@ theorem coe_zero : ((0 : AlternatingMap R M N ι) : MultilinearMap R (fun _ : ι
rfl
#align alternating_map.coe_zero AlternatingMap.coe_zero

@[simp]
theorem mk_zero :
mk (0 : MultilinearMap R (fun _ : ι ↦ M) N) (0 : AlternatingMap R M N ι).2 = 0 :=
rfl

instance inhabited : Inhabited (AlternatingMap R M N ι) :=
0
#align alternating_map.inhabited AlternatingMap.inhabited
Expand Down

0 comments on commit a691787

Please sign in to comment.