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

Commit c63caeb

Browse files
committed
feat(algebra/homology): homotopies between chain maps (#7483)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent cc47aff commit c63caeb

File tree

2 files changed

+500
-1
lines changed

2 files changed

+500
-1
lines changed

src/algebra/homology/additive.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -41,7 +41,6 @@ instance : has_sub (C ⟶ D) := ⟨λ f g, { f := λ i, f.f i - g.f i, }⟩
4141
@[simp] lemma neg_f_apply (f : C ⟶ D) (i : ι) : (-f).f i = -(f.f i) := rfl
4242
@[simp] lemma sub_f_apply (f g : C ⟶ D) (i : ι) : (f - g).f i = f.f i - g.f i := rfl
4343

44-
4544
/- TODO(jmc/Scott): the instance below doesn't have the correct defeq for `nsmul` and `gsmul`.
4645
We should generalize `function.injective.add_comm_group` and friends.
4746
For the `R`-linear version, it will be very convenient to have

0 commit comments

Comments
 (0)