Skip to content

Commit

Permalink
fix test
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Feb 4, 2025
1 parent c2681ef commit 51879e1
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
4 changes: 2 additions & 2 deletions test/Mathlib/test/H20231020.in
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@

{"cmd": "theorem mathd_numbertheory_188 : Nat.gcd 180 168 = 12 := by norm_num", "env": 0}

{"cmd": "theorem mathd_numbertheory_403 : ∑ k in (Nat.properDivisors 198), k = 270 := by simp (config := {decide := true})", "env": 0}
{"cmd": "theorem mathd_numbertheory_403 : ∑ k (Nat.properDivisors 198), k = 270 := by simp (config := {decide := true})", "env": 0}

{"cmd": "theorem mathd_numbertheory_109 (v : ℕ → ℕ) (h₀ : ∀ n, v n = 2 * n - 1) : (∑ k in Finset.Icc 1 100, v k) % 7 = 4 := by simp_rw (config := {decide := true}) [h₀]", "env": 0}
{"cmd": "theorem mathd_numbertheory_109 (v : ℕ → ℕ) (h₀ : ∀ n, v n = 2 * n - 1) : (∑ k Finset.Icc 1 100, v k) % 7 = 4 := by simp_rw (config := {decide := true}) [h₀]", "env": 0}

4 changes: 2 additions & 2 deletions test/Mathlib/test/H20231020.lean
Original file line number Diff line number Diff line change
Expand Up @@ -17,6 +17,6 @@ open Topology

theorem mathd_numbertheory_188 : Nat.gcd 180 168 = 12 := by norm_num

theorem mathd_numbertheory_403 : ∑ k in (Nat.properDivisors 198), k = 270 := by simp (config := {decide := true})
theorem mathd_numbertheory_403 : ∑ k (Nat.properDivisors 198), k = 270 := by simp (config := {decide := true})

theorem mathd_numbertheory_109 (v : ℕ → ℕ) (h₀ : ∀ n, v n = 2 * n - 1) : (∑ k in Finset.Icc 1 100, v k) % 7 = 4 := by simp_rw (config := {decide := true}) [h₀]
theorem mathd_numbertheory_109 (v : ℕ → ℕ) (h₀ : ∀ n, v n = 2 * n - 1) : (∑ k Finset.Icc 1 100, v k) % 7 = 4 := by simp_rw (config := {decide := true}) [h₀]

0 comments on commit 51879e1

Please sign in to comment.