Skip to content

Commit

Permalink
chore: remove references to fixed lean bug (#1338)
Browse files Browse the repository at this point in the history
Followup to #1335.
  • Loading branch information
Ruben-VandeVelde committed Jan 4, 2023
1 parent 7e2613a commit c0e8ec7
Show file tree
Hide file tree
Showing 3 changed files with 0 additions and 3 deletions.
1 change: 0 additions & 1 deletion Mathlib/Order/Antichain.lean
Expand Up @@ -336,7 +336,6 @@ variable {ι : Type _} {α : ι → Type _} [∀ i, Preorder (α i)] {s t : Set
{a b c : ∀ i, α i}


-- Porting note: local notation given a name because of https://github.com/leanprover/lean4/issues/2000
@[inherit_doc]
local infixl:50 " ≺ " => StrongLT

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Order/Chain.lean
Expand Up @@ -44,7 +44,6 @@ section Chain
variable (r : α → α → Prop)

/-- In this file, we use `≺` as a local notation for any relation `r`. -/
-- Porting note: local notation given a name because of https://github.com/leanprover/lean4/issues/2000
local infixl:50 " ≺ " => r

/-- A chain is a set `s` satisfying `x ≺ y ∨ x = y ∨ y ≺ x` for all `x y ∈ s`. -/
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Order/Zorn.lean
Expand Up @@ -71,7 +71,6 @@ open Classical Set
variable {α β : Type _} {r : α → α → Prop} {c : Set α}

/-- Local notation for the relation being considered. -/
-- Porting note: local notation given a name because of https://github.com/leanprover/lean4/issues/2000
local infixl:50 " ≺ " => r

/-- **Zorn's lemma**
Expand Down

0 comments on commit c0e8ec7

Please sign in to comment.