Skip to content

Commit c91c157

Browse files
committed
chore(Order/Defs/PartialOrder): fix typo in decidableEqofDecidableLE' (#31857)
This is a follow-up to #31816, fixing another typo in the same declaration. decidableEqofDecidableLE' -> decidableEqOfDecidableLE'
1 parent f7442dd commit c91c157

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Order/Defs/PartialOrder.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -206,7 +206,7 @@ lemma lt_of_le_of_ne : a ≤ b → a ≠ b → a < b := fun h₁ h₂ =>
206206
lt_of_le_not_ge h₁ <| mt (le_antisymm h₁) h₂
207207

208208
/-- Equality is decidable if `≤` is. -/
209-
@[to_dual decidableEqofDecidableLE' /-- Equality is decidable if `≤` is. -/]
209+
@[to_dual decidableEqOfDecidableLE' /-- Equality is decidable if `≤` is. -/]
210210
def decidableEqOfDecidableLE [DecidableLE α] : DecidableEq α
211211
| a, b =>
212212
if hab : a ≤ b then

0 commit comments

Comments
 (0)