src/HOL/Homology/Simplices.thy
changeset 73655 26a1d66b9077
parent 72794 3757e64e75bb
child 73869 7181130f5872
child 73932 fd21b4a93043
--- a/src/HOL/Homology/Simplices.thy	Mon May 10 14:28:37 2021 +0200
+++ b/src/HOL/Homology/Simplices.thy	Mon May 10 16:14:34 2021 +0200
@@ -2347,7 +2347,8 @@
     show "chain_boundary (Suc p) (?h p c) + ?h (p - Suc 0) (chain_boundary p c) = (singular_subdivision p ^^ Suc n) c - c"
       using chain_boundary_singular_subdivision [of "Suc p" X]
       apply (simp add: chain_boundary_add f5 h k algebra_simps)
-      by (smt add.assoc add.commute diff_add_cancel h(4) k(4) sc singular_subdivision_add)
+      apply (smt (verit, ccfv_threshold) add.commute add_diff_eq diff_add_cancel diff_diff_eq2 h(4) k(4) sc singular_subdivision_add)
+      done
   qed (auto simp: k h singular_subdivision_diff)
 qed