Skip to content

Commit 40b85e9

Browse files
wuprkbuzzard
authored andcommitted
fix: rename orderOf_mk to Prod.orderOf_mk (#14154)
1 parent c5a66cd commit 40b85e9

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/GroupTheory/OrderOfElement.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -1304,7 +1304,7 @@ theorem IsOfFinOrder.prod_mk : IsOfFinOrder a → IsOfFinOrder b → IsOfFinOrde
13041304
#align is_of_fin_add_order.prod_mk IsOfFinAddOrder.prod_mk
13051305

13061306
@[to_additive]
1307-
lemma orderOf_mk {a : α} {b : β} : orderOf (a, b) = Nat.lcm (orderOf a) (orderOf b) :=
1307+
lemma Prod.orderOf_mk : orderOf (a, b) = Nat.lcm (orderOf a) (orderOf b) :=
13081308
(a, b).orderOf
13091309

13101310
end Prod

0 commit comments

Comments
 (0)