Skip to content

Commit

Permalink
suggestions from review
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jan 5, 2025
1 parent 0c2797e commit fc67869
Show file tree
Hide file tree
Showing 3 changed files with 2 additions and 5 deletions.
1 change: 0 additions & 1 deletion Mathlib/Algebra/Category/ModuleCat/Subobject.lean
Original file line number Diff line number Diff line change
Expand Up @@ -85,7 +85,6 @@ theorem toKernelSubobject_arrow {M N : ModuleCat R} {f : M ⟶ N} (x : LinearMap
suffices ((arrow ((kernelSubobject f))) ∘ (kernelSubobjectIso f ≪≫ kernelIsoKer f).inv) x = x by
convert this
rw [Iso.trans_inv, ← LinearMap.coe_comp, ← hom_comp, Category.assoc]
simp only [Category.assoc, kernelSubobject_arrow', kernelIsoKer_inv_kernel_ι]
simp

/-- An extensionality lemma showing that two elements of a cokernel by an image
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/Data/Matrix/ColumnRowPartitioned.lean
Original file line number Diff line number Diff line change
Expand Up @@ -125,8 +125,7 @@ lemma fromRows_toRows (A : Matrix (m₁ ⊕ m₂) n R) : fromRows A.toRows₁ A.

lemma fromRows_inj : Function.Injective2 (@fromRows R m₁ m₂ n) := by
intros x1 x2 y1 y2
simp only [funext_iff, ← Matrix.ext_iff]
simp
simp [← Matrix.ext_iff]

lemma fromCols_inj : Function.Injective2 (@fromCols R m n₁ n₂) := by
intros x1 x2 y1 y2
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/LinearAlgebra/Semisimple.lean
Original file line number Diff line number Diff line change
Expand Up @@ -73,8 +73,7 @@ lemma isSemisimple_iff' :

lemma isSemisimple_iff :
f.IsSemisimple ↔ ∀ p ∈ invtSubmodule f, ∃ q ∈ invtSubmodule f, IsCompl p q := by
simp_rw [isSemisimple_iff']
simp
simp [isSemisimple_iff']

lemma isSemisimple_restrict_iff (p) (hp : p ∈ invtSubmodule f) :
IsSemisimple (LinearMap.restrict f hp) ↔
Expand Down

0 comments on commit fc67869

Please sign in to comment.