Skip to content

Commit 4481ab6

Browse files
committed
deprecations
1 parent b1ccddb commit 4481ab6

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

Mathlib/Algebra/Homology/HomotopyCategory/HomComplexCohomology.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -46,7 +46,7 @@ def coboundaries : AddSubgroup (Cocycle K L n) where
4646
zero_mem' := ⟨n - 1, by simp, 0, by simp⟩
4747
add_mem' := by
4848
rintro α₁ α₂ ⟨m, hm, β₁, hβ₁⟩ ⟨m', hm', β₂, hβ₂⟩
49-
obtain rfl : m = m' := by cutsat
49+
obtain rfl : m = m' := by lia
5050
exact ⟨m, hm, β₁ + β₂, by aesop⟩
5151
neg_mem' := by
5252
rintro α ⟨m, hm, β, hβ⟩
@@ -138,7 +138,7 @@ def leftHomologyData' (hm : n + 1 = m) (hp : m + 1 = p) :
138138
(fun s ↦ AddCommGrpCat.ofHom (CohomologyClass.descAddMonoidHom s.π.hom
139139
(by
140140
rintro ⟨_, _⟩ ⟨q, hq, y, rfl⟩
141-
obtain rfl : n = q := by cutsat
141+
obtain rfl : n = q := by lia
142142
simpa only [zero_comp] using ConcreteCategory.congr_hom s.condition y)))
143143
(fun s ↦ rfl)
144144
(fun s l hl ↦ by

0 commit comments

Comments
 (0)