Skip to content

Commit

Permalink
docs
Browse files Browse the repository at this point in the history
  • Loading branch information
jjaassoonn committed Jul 8, 2024
1 parent 86c2dee commit 32f3feb
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion Mathlib/RingTheory/Flat/CategoryTheory.lean
Original file line number Diff line number Diff line change
Expand Up @@ -165,7 +165,7 @@ section Tor

open scoped ZeroObject

/-
/--
For a flat module `M`, higher tor groups vanish.
-/
noncomputable def higherTorIsoZero [Flat R M] (n : ℕ) (N : ModuleCat.{u} R) :
Expand All @@ -187,6 +187,7 @@ noncomputable def higherTor'IsoZero [Flat R M] (n : ℕ) (N : ModuleCat.{u} R) :
rTensor_shortComplex_exact M (pN.complex.sc (n + 1)) (pN.complex_exactAt_succ n))



end Tor

end Module.Flat

0 comments on commit 32f3feb

Please sign in to comment.