Skip to content

Commit

Permalink
fix: correct doc-string for LocallyFiniteOrderTop/Bot (#5956)
Browse files Browse the repository at this point in the history
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Jul 19, 2023
1 parent 26d0eab commit 9b5b824
Showing 1 changed file with 5 additions and 4 deletions.
9 changes: 5 additions & 4 deletions Mathlib/Order/LocallyFinite.lean
Expand Up @@ -110,8 +110,9 @@ as `Icc (-1) 1` is infinite.

open Finset Function

/-- A locally finite order is an order where bounded intervals are finite. When you don't care too
much about definitional equality, you can use `LocallyFiniteOrder.ofIcc` or
/-- This is a mixin class describing a locally finite order,
that is, is an order where bounded intervals are finite.
When you don't care too much about definitional equality, you can use `LocallyFiniteOrder.ofIcc` or
`LocallyFiniteOrder.ofFiniteIcc` to build a locally finite order from just `Finset.Icc`. -/
class LocallyFiniteOrder (α : Type _) [Preorder α] where
/-- Left-closed right-closed interval -/
Expand All @@ -132,7 +133,7 @@ class LocallyFiniteOrder (α : Type _) [Preorder α] where
finset_mem_Ioo : ∀ a b x : α, x ∈ finsetIoo a b ↔ a < x ∧ x < b
#align locally_finite_order LocallyFiniteOrder

/-- A locally finite order top is an order where all intervals bounded above are finite. This is
/-- This mixin class describes an order where all intervals bounded below are finite. This is
slightly weaker than `LocallyFiniteOrder` + `OrderTop` as it allows empty types. -/
class LocallyFiniteOrderTop (α : Type _) [Preorder α] where
/-- Left-open right-infinite interval -/
Expand All @@ -145,7 +146,7 @@ class LocallyFiniteOrderTop (α : Type _) [Preorder α] where
finset_mem_Ioi : ∀ a x : α, x ∈ finsetIoi a ↔ a < x
#align locally_finite_order_top LocallyFiniteOrderTop

/-- A locally finite order bot is an order where all intervals bounded below are finite. This is
/-- This mixin class describes an order where all intervals bounded above are finite. This is
slightly weaker than `LocallyFiniteOrder` + `OrderBot` as it allows empty types. -/
class LocallyFiniteOrderBot (α : Type _) [Preorder α] where
/-- Left-infinite right-open interval -/
Expand Down

0 comments on commit 9b5b824

Please sign in to comment.