Skip to content

Commit 4f1434c

Browse files
committed
fix tests
1 parent 1e86f81 commit 4f1434c

File tree

3 files changed

+5
-4
lines changed

3 files changed

+5
-4
lines changed

src/Init/Data/Fin/Lemmas.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1137,6 +1137,7 @@ theorem mul_ofNat [NeZero n] (x : Fin n) (y : Nat) :
11371137
theorem val_mul {n : Nat} : ∀ a b : Fin n, (a * b).val = a.val * b.val % n
11381138
| ⟨_, _⟩, ⟨_, _⟩ => rfl
11391139

1140+
@[deprecated val_mul (since := "2025-10-26")]
11401141
theorem coe_mul {n : Nat} : ∀ a b : Fin n, ((a * b : Fin n) : Nat) = a * b % n
11411142
| ⟨_, _⟩, ⟨_, _⟩ => rfl
11421143

tests/lean/run/symbolFrequency.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,4 +7,4 @@ open Lean PremiseSelection
77
#guard_msgs in
88
run_meta do
99
let f ← symbolFrequency `Nat
10-
logInfo m!"{decide (10000 < f)}"
10+
logInfo m!"{decide (5000 < f)}"

tests/lean/run/symbolFrequency_foldRelevantConsts.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -9,19 +9,19 @@ open Lean PremiseSelection
99
#guard_msgs in
1010
run_meta do
1111
let ci ← getConstInfo `List.append_assoc
12-
let consts ← foldRelevantConsts ci.type (init := #[]) (fun n ns => return ns.push n)
12+
let consts ← ci.type.foldRelevantConstants (init := #[]) (fun n ns => return ns.push n)
1313
logInfo m!"{consts}"
1414

1515
/-- info: [List, Ne, HAppend.hAppend, List.nil, Eq, List.head] -/
1616
#guard_msgs in
1717
run_meta do
1818
let ci ← getConstInfo `List.head_append_right
19-
let consts ← foldRelevantConsts ci.type (init := #[]) (fun n ns => return ns.push n)
19+
let consts ← ci.type.foldRelevantConstants (init := #[]) (fun n ns => return ns.push n)
2020
logInfo m!"{consts}"
2121

2222
/-- info: [Array, Nat, LT.lt, Array.size, HAdd.hAdd, OfNat.ofNat, Array.swap, Not] -/
2323
#guard_msgs in
2424
run_meta do
2525
let ci ← getConstInfo `Array.eraseIdx.induct
26-
let consts ← foldRelevantConsts ci.type (init := #[]) (fun n ns => return ns.push n)
26+
let consts ← ci.type.foldRelevantConstants (init := #[]) (fun n ns => return ns.push n)
2727
logInfo m!"{consts}"

0 commit comments

Comments
 (0)