Skip to content

Commit

Permalink
feat(algebra/homology): homotopies between chain maps (#7483)
Browse files Browse the repository at this point in the history
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed May 15, 2021
1 parent cc47aff commit c63caeb
Show file tree
Hide file tree
Showing 2 changed files with 500 additions and 1 deletion.
1 change: 0 additions & 1 deletion src/algebra/homology/additive.lean
Expand Up @@ -41,7 +41,6 @@ instance : has_sub (C ⟶ D) := ⟨λ f g, { f := λ i, f.f i - g.f i, }⟩
@[simp] lemma neg_f_apply (f : C ⟶ D) (i : ι) : (-f).f i = -(f.f i) := rfl
@[simp] lemma sub_f_apply (f g : C ⟶ D) (i : ι) : (f - g).f i = f.f i - g.f i := rfl


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

0 comments on commit c63caeb

Please sign in to comment.