Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit bd65478

Browse files
committed
chore(linear_algebra/alternating): make ι an explicit arg of alternating_map.const_of_is_empty (#19123)
While for general multilinear maps one can deduce it from the type of `E : ι -> Type*`, this doesn't work for alternating maps.
1 parent 837f72d commit bd65478

File tree

3 files changed

+5
-3
lines changed

3 files changed

+5
-3
lines changed

src/analysis/inner_product_space/orientation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -181,7 +181,7 @@ alternating form uniquely defined by compatibility with the orientation and inne
181181
begin
182182
classical,
183183
unfreezingI { cases n },
184-
{ let opos : alternating_map ℝ E ℝ (fin 0) := alternating_map.const_of_is_empty ℝ E (1:ℝ),
184+
{ let opos : alternating_map ℝ E ℝ (fin 0) := alternating_map.const_of_is_empty ℝ E (fin 0) (1:ℝ),
185185
exact o.eq_or_eq_neg_of_is_empty.by_cases (λ _, opos) (λ _, -opos) },
186186
{ exact (o.fin_orthonormal_basis n.succ_pos _i.out).to_basis.det }
187187
end

src/linear_algebra/alternating.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -337,6 +337,8 @@ def of_subsingleton [subsingleton ι] (i : ι) : alternating_map R M M ι :=
337337
map_eq_zero_of_eq' := λ v i j hv hij, (hij $ subsingleton.elim _ _).elim,
338338
..multilinear_map.of_subsingleton R M i }
339339

340+
variable (ι)
341+
340342
/-- The constant map is alternating when `ι` is empty. -/
341343
@[simps {fully_applied := ff}]
342344
def const_of_is_empty [is_empty ι] (m : N) : alternating_map R M N ι :=
@@ -1102,7 +1104,7 @@ end
11021104
to an empty family. -/
11031105
@[simps] def const_linear_equiv_of_is_empty [is_empty ι] :
11041106
N'' ≃ₗ[R'] alternating_map R' M'' N'' ι :=
1105-
{ to_fun := alternating_map.const_of_is_empty R' M'',
1107+
{ to_fun := alternating_map.const_of_is_empty R' M'' ι,
11061108
map_add' := λ x y, rfl,
11071109
map_smul' := λ t x, rfl,
11081110
inv_fun := λ f, f 0,

src/linear_algebra/determinant.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -480,7 +480,7 @@ lemma basis.det_apply (v : ι → M) : e.det v = det (e.to_matrix v) := rfl
480480
lemma basis.det_self : e.det e = 1 :=
481481
by simp [e.det_apply]
482482

483-
@[simp] lemma basis.det_is_empty [is_empty ι] : e.det = alternating_map.const_of_is_empty R M 1 :=
483+
@[simp] lemma basis.det_is_empty [is_empty ι] : e.det = alternating_map.const_of_is_empty R M ι 1 :=
484484
begin
485485
ext v,
486486
exact matrix.det_is_empty,

0 commit comments

Comments
 (0)