Skip to content

Commit bf1dbb9

Browse files
committed
chore(Order/Defs): golf min_def (#30924)
After this change, `min_def` has a proof term that indicates that it is an alias of `LinearOrder.min_def`. So the duplicate declaration linter will not report it.
1 parent 9b82ea7 commit bf1dbb9

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

Mathlib/Order/Defs/LinearOrder.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -133,9 +133,9 @@ theorem le_imp_le_of_lt_imp_lt {α β} [Preorder α] [LinearOrder β] {a b : α}
133133
le_of_not_gt fun h' => not_le_of_gt (H h') h
134134

135135
@[grind =]
136-
lemma min_def (a b : α) : min a b = if a ≤ b then a else b := by rw [LinearOrder.min_def a]
136+
lemma min_def (a b : α) : min a b = if a ≤ b then a else b := LinearOrder.min_def a b
137137
@[grind =]
138-
lemma max_def (a b : α) : max a b = if a ≤ b then b else a := by rw [LinearOrder.max_def a]
138+
lemma max_def (a b : α) : max a b = if a ≤ b then b else a := LinearOrder.max_def a b
139139

140140
lemma min_le_left (a b : α) : min a b ≤ a := by
141141
if h : a ≤ b

0 commit comments

Comments
 (0)