Skip to content

Commit

Permalink
remove lemma
Browse files Browse the repository at this point in the history
  • Loading branch information
vasnesterov committed Feb 15, 2025
1 parent 8ef7ffe commit 9918a87
Showing 1 changed file with 3 additions and 6 deletions.
9 changes: 3 additions & 6 deletions Mathlib/Tactic/Order.lean
Original file line number Diff line number Diff line change
Expand Up @@ -208,9 +208,6 @@ where

section Preprocessing

private lemma le_of_eq_symm {α : Type} [Preorder α] {x y : α} (h : x = y) : y ≤ x :=
ge_of_eq h

private lemma not_lt_of_not_le {α : Type} [Preorder α] {x y : α} (h : ¬(x ≤ y)) : ¬(x < y) := by
intro h'
exact h h'.le
Expand All @@ -234,7 +231,7 @@ def preprocessFactsPreorder (g : MVarId) (facts : Array AtomicFact) :
res := res.push ⟨fact.rhs, fact.lhs, .nle, ← mkAppM ``not_le_of_lt #[fact.proof]⟩
| .eq =>
res := res.push ⟨fact.lhs, fact.rhs, .le, ← mkAppM ``le_of_eq #[fact.proof]⟩
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``le_of_eq_symm #[fact.proof]⟩
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``ge_of_eq #[fact.proof]⟩
| .ne =>
continue
| _ =>
Expand All @@ -256,7 +253,7 @@ def preprocessFactsPartial (g : MVarId) (facts : Array AtomicFact) :
res := res.push ⟨fact.lhs, fact.rhs, .nlt, ← mkAppM ``not_lt_of_not_le #[fact.proof]⟩
| .eq =>
res := res.push ⟨fact.lhs, fact.rhs, .le, ← mkAppM ``le_of_eq #[fact.proof]⟩
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``le_of_eq_symm #[fact.proof]⟩
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``ge_of_eq #[fact.proof]⟩
| _ =>
res := res.push fact
return res
Expand All @@ -278,7 +275,7 @@ def preprocessFactsLinear (g : MVarId) (facts : Array AtomicFact) :
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``le_of_not_lt #[fact.proof]⟩
| .eq =>
res := res.push ⟨fact.lhs, fact.rhs, .le, ← mkAppM ``le_of_eq #[fact.proof]⟩
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``le_of_eq_symm #[fact.proof]⟩
res := res.push ⟨fact.rhs, fact.lhs, .le, ← mkAppM ``ge_of_eq #[fact.proof]⟩
| _ =>
res := res.push fact
return res
Expand Down

0 comments on commit 9918a87

Please sign in to comment.