Skip to content

Commit 3dc572b

Browse files
committed
grind +revert
1 parent 37c4d0a commit 3dc572b

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -540,7 +540,7 @@ lemma liftCochain_descCochain :
540540
lemma liftCochain_v_descCochain_v (p₁ p₂ p₃ : ℤ) (h₁₂ : p₁ + n = p₂) (h₂₃ : p₂ + n' = p₃)
541541
(q : ℤ) (hq : p₁ + m = q) :
542542
(liftCochain φ α β h).v p₁ p₂ h₁₂ ≫ (descCochain φ α' β' h').v p₂ p₃ h₂₃ =
543-
α.v p₁ q hq ≫ α'.v q p₃ (by cutsat) + β.v p₁ p₂ h₁₂ ≫ β'.v p₂ p₃ h₂₃ := by
543+
α.v p₁ q hq ≫ α'.v q p₃ (by grind +revert) + β.v p₁ p₂ h₁₂ ≫ β'.v p₂ p₃ h₂₃ := by
544544
have eq := Cochain.congr_v (liftCochain_descCochain φ α β α' β' h h' p hp) p₁ p₃ (by cutsat)
545545
simpa only [Cochain.comp_v _ _ hp p₁ p₂ p₃ h₁₂ h₂₃, Cochain.add_v,
546546
Cochain.comp_v _ _ _ _ _ _ hq (show q + m' = p₃ by cutsat)] using eq

Mathlib/Algebra/Ring/GeomSum.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@ lemma op_geom_sum₂ (x y : R) (n : ℕ) : ∑ i ∈ range n, op y ^ (n - 1 - i)
6565
∑ i ∈ range n, op y ^ i * op x ^ (n - 1 - i) := by
6666
rw [← sum_range_reflect]
6767
refine sum_congr rfl fun j j_in => ?_
68-
grind
68+
grind +revert
6969

7070
lemma geom_sum₂_with_one (x : R) (n : ℕ) :
7171
∑ i ∈ range n, x ^ i * 1 ^ (n - 1 - i) = ∑ i ∈ range n, x ^ i :=

0 commit comments

Comments
 (0)