Skip to content

Commit 6c406a5

Browse files
committed
cutsat to lia
1 parent a7967a1 commit 6c406a5

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

Mathlib/CategoryTheory/Shift/CommShiftTwo.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -66,7 +66,7 @@ noncomputable def CommShift₂Setup.int [Preadditive D] [HasShift D ℤ]
6666
assoc _ _ _ := by
6767
dsimp
6868
rw [← zpow_add, ← zpow_add]
69-
cutsat
69+
lia
7070
commShift _ _ := ⟨by cat_disch⟩
7171
ε p q := (-1) ^ (p * q)
7272

Mathlib/RingTheory/IntegralClosure/Algebra/Ideal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -96,7 +96,7 @@ lemma exists_monic_aeval_eq_zero_forall_mem_of_mem_map [Algebra.IsIntegral R S]
9696
obtain ⟨p, hp, e, h⟩ := exists_monic_aeval_eq_zero_forall_mem_pow_of_mem_map hx
9797
refine ⟨p, hp, e, fun i hi ↦ ?_⟩
9898
obtain hi | hi := hi.lt_or_gt
99-
· exact Ideal.pow_le_self (by cutsat) (h _)
99+
· exact Ideal.pow_le_self (by lia) (h _)
100100
· simp [coeff_eq_zero_of_natDegree_lt hi]
101101

102102
end Polynomial

0 commit comments

Comments
 (0)