mathlib3 documentation

data.set.intervals.infinite

Infinitude of intervals #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Bounded intervals in dense orders are infinite, as are unbounded intervals in orders that are unbounded on the appropriate side. We also prove that an unbounded preorder is an infinite type.

theorem no_max_order.infinite {α : Type u_1} [preorder α] [nonempty α] [no_max_order α] :

A nonempty preorder with no maximal element is infinite. This is not an instance to avoid a cycle with infinite α → nontrivial α → nonempty α.

theorem no_min_order.infinite {α : Type u_1} [preorder α] [nonempty α] [no_min_order α] :

A nonempty preorder with no minimal element is infinite. This is not an instance to avoid a cycle with infinite α → nontrivial α → nonempty α.

theorem set.Ioo.infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Ioo_infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Ico_infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Ico.infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Ioc_infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Ioc.infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Icc_infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
theorem set.Icc.infinite {α : Type u_1} [preorder α] [densely_ordered α] {a b : α} (h : a < b) :
@[protected, instance]
def set.Iio.infinite {α : Type u_1} [preorder α] [no_min_order α] {a : α} :
theorem set.Iio_infinite {α : Type u_1} [preorder α] [no_min_order α] (a : α) :
@[protected, instance]
def set.Iic.infinite {α : Type u_1} [preorder α] [no_min_order α] {a : α} :
theorem set.Iic_infinite {α : Type u_1} [preorder α] [no_min_order α] (a : α) :
@[protected, instance]
def set.Ioi.infinite {α : Type u_1} [preorder α] [no_max_order α] {a : α} :
theorem set.Ioi_infinite {α : Type u_1} [preorder α] [no_max_order α] (a : α) :
@[protected, instance]
def set.Ici.infinite {α : Type u_1} [preorder α] [no_max_order α] {a : α} :
theorem set.Ici_infinite {α : Type u_1} [preorder α] [no_max_order α] (a : α) :