Skip to content

Commit

Permalink
refactor(algebra/category/Group/limits): simp -> refl (#5911)
Browse files Browse the repository at this point in the history
Co-authors: `lean-gptf`, Stanislas Polu
  • Loading branch information
Jesse Michael Han committed Jan 27, 2021
1 parent 6eae630 commit 38f6e05
Showing 1 changed file with 1 addition and 4 deletions.
5 changes: 1 addition & 4 deletions src/algebra/category/Group/limits.lean
Expand Up @@ -247,10 +247,7 @@ def kernel_iso_ker {G H : AddCommGroup} (f : G ⟶ H) :
@[simp]
lemma kernel_iso_ker_hom_comp_subtype {G H : AddCommGroup} (f : G ⟶ H) :
(kernel_iso_ker f).hom ≫ add_subgroup.subtype f.ker = kernel.ι f :=
begin
ext,
simp [kernel_iso_ker],
end
by ext; refl

@[simp]
lemma kernel_iso_ker_inv_comp_ι {G H : AddCommGroup} (f : G ⟶ H) :
Expand Down

0 comments on commit 38f6e05

Please sign in to comment.