Skip to content

Commit ae4dd74

Browse files
chore: remove redundant LinearEquiv.map_neg/sub (#12330)
These are redundant with `_root_.{map_neg,map_sub}`.
1 parent a9cdcd2 commit ae4dd74

File tree

6 files changed

+9
-16
lines changed

6 files changed

+9
-16
lines changed

Mathlib/Algebra/Lie/Matrix.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -45,7 +45,7 @@ def lieEquivMatrix' : Module.End R (n → R) ≃ₗ⁅R⁆ Matrix n n R :=
4545
let f := @LinearMap.toMatrix' R _ n n _ _
4646
change f (T.comp S - S.comp T) = f T * f S - f S * f T
4747
have h : ∀ T S : Module.End R _, f (T.comp S) = f T * f S := LinearMap.toMatrix'_comp
48-
rw [LinearEquiv.map_sub, h, h] }
48+
rw [map_sub, h, h] }
4949
#align lie_equiv_matrix' lieEquivMatrix'
5050

5151
@[simp]

Mathlib/Algebra/Lie/OfAssociative.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -377,7 +377,7 @@ def lieConj : Module.End R M₁ ≃ₗ⁅R⁆ Module.End R M₂ :=
377377
map_lie' := fun {f g} =>
378378
show e.conj ⁅f, g⁆ = ⁅e.conj f, e.conj g⁆ by
379379
simp only [LieRing.of_associative_ring_bracket, LinearMap.mul_eq_comp, e.conj_comp,
380-
LinearEquiv.map_sub] }
380+
map_sub] }
381381
#align linear_equiv.lie_conj LinearEquiv.lieConj
382382

383383
@[simp]

Mathlib/Algebra/Module/Zlattice/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -145,7 +145,7 @@ theorem fract_apply (m : E) : fract b m = m - floor b m := rfl
145145

146146
@[simp]
147147
theorem repr_fract_apply (m : E) (i : ι) : b.repr (fract b m) i = Int.fract (b.repr m i) := by
148-
rw [fract, LinearEquiv.map_sub, Finsupp.coe_sub, Pi.sub_apply, repr_floor_apply, Int.fract]
148+
rw [fract, map_sub, Finsupp.coe_sub, Pi.sub_apply, repr_floor_apply, Int.fract]
149149
#align zspan.repr_fract_apply Zspan.repr_fract_apply
150150

151151
@[simp]
@@ -195,7 +195,7 @@ theorem fract_eq_fract (m n : E) : fract b m = fract b n ↔ -m + n ∈ span ℤ
195195
classical
196196
rw [eq_comm, Basis.ext_elem_iff b]
197197
simp_rw [repr_fract_apply, Int.fract_eq_fract, eq_comm, Basis.mem_span_iff_repr_mem,
198-
sub_eq_neg_add, map_add, LinearEquiv.map_neg, Finsupp.coe_add, Finsupp.coe_neg, Pi.add_apply,
198+
sub_eq_neg_add, map_add, map_neg, Finsupp.coe_add, Finsupp.coe_neg, Pi.add_apply,
199199
Pi.neg_apply, ← eq_intCast (algebraMap ℤ K) _, Set.mem_range]
200200
#align zspan.fract_eq_fract Zspan.fract_eq_fract
201201

Mathlib/LinearAlgebra/Basic.lean

Lines changed: 2 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -532,15 +532,8 @@ variable {re₁₂ : RingHomInvPair σ₁₂ σ₂₁} {re₂₁ : RingHomInvPai
532532
variable {re₃₄ : RingHomInvPair σ₃₄ σ₄₃} {re₄₃ : RingHomInvPair σ₄₃ σ₃₄}
533533
variable (e e₁ : M ≃ₛₗ[σ₁₂] M₂) (e₂ : M₃ ≃ₛₗ[σ₃₄] M₄)
534534

535-
-- @[simp] -- Porting note (#10618): simp can prove this
536-
theorem map_neg (a : M) : e (-a) = -e a :=
537-
e.toLinearMap.map_neg a
538-
#align linear_equiv.map_neg LinearEquiv.map_neg
539-
540-
-- @[simp] -- Porting note (#10618): simp can prove this
541-
theorem map_sub (a b : M) : e (a - b) = e a - e b :=
542-
e.toLinearMap.map_sub a b
543-
#align linear_equiv.map_sub LinearEquiv.map_sub
535+
#align linear_equiv.map_neg map_negₓ
536+
#align linear_equiv.map_sub map_subₓ
544537

545538
end AddCommGroup
546539

Mathlib/LinearAlgebra/Basis.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1573,8 +1573,8 @@ theorem union_support_maximal_linearIndependent_eq_range_basis {ι : Type w} (b
15731573
rw [← eq_neg_iff_add_eq_zero] at z
15741574
replace z := neg_eq_iff_eq_neg.mpr z
15751575
apply_fun fun x => b.repr x b' at z
1576-
simp only [repr_self, LinearEquiv.map_smul, mul_one, Finsupp.single_eq_same, Pi.neg_apply,
1577-
Finsupp.smul_single', LinearEquiv.map_neg, Finsupp.coe_neg] at z
1576+
simp only [repr_self, map_smul, mul_one, Finsupp.single_eq_same, Pi.neg_apply,
1577+
Finsupp.smul_single', map_neg, Finsupp.coe_neg] at z
15781578
erw [DFunLike.congr_fun (Finsupp.apply_total R (b.repr : M →ₗ[R] ι →₀ R) v l.some) b'] at z
15791579
simpa [Finsupp.total_apply, w] using z
15801580
-- Then all the other coefficients are zero, because `v` is linear independent.

Mathlib/NumberTheory/ClassNumber/Finite.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -246,7 +246,7 @@ theorem exists_mem_finsetApprox (a : S) {b} (hb : b ≠ (0 : R)) :
246246
refine' Int.cast_lt.mp ((norm_lt abv bS _ fun i => lt_of_le_of_lt _ (hjk' i)).trans_le _)
247247
· apply le_of_eq
248248
congr
249-
simp_rw [map_sum, LinearEquiv.map_sub, LinearEquiv.map_smul, Finset.sum_apply',
249+
simp_rw [map_sum, map_sub, map_smul, Finset.sum_apply',
250250
Finsupp.sub_apply, Finsupp.smul_apply, Finset.sum_sub_distrib, Basis.repr_self_apply,
251251
smul_eq_mul, mul_boole, Finset.sum_ite_eq', Finset.mem_univ, if_true]
252252
· exact mod_cast ε_le

0 commit comments

Comments
 (0)