Skip to content

Commit 38865c5

Browse files
committed
fix deprecation
1 parent 905c960 commit 38865c5

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Init/Data/Fin/Lemmas.lean

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

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

0 commit comments

Comments
 (0)