Intervals Ixx (f x) (f (order.succ x))
#
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove
-
monotone.bUnion_Ico_Ioc_map_succ
: ifα
is a linear archimedean succ order andβ
is a linear order, then for any monotone functionf
andm n : α
, the union of intervalsset.Ioc (f i) (f (order.succ i))
,m ≤ i < n
, is equal toset.Ioc (f m) (f n)
; -
monotone.pairwise_disjoint_on_Ioc_succ
: ifα
is a linear succ order,β
is a preorder, andf : α → β
is a monotone function, then the intervalsset.Ioc (f n) (f (order.succ n))
are pairwise disjoint.
For the latter lemma, we also prove various order dual versions.
If α
is a linear archimedean succ order and β
is a linear order, then for any monotone
function f
and m n : α
, the union of intervals set.Ioc (f i) (f (order.succ i))
, m ≤ i < n
,
is equal to set.Ioc (f m) (f n)
If α
is a linear succ order, β
is a preorder, and f : α → β
is a monotone function, then
the intervals set.Ioc (f n) (f (order.succ n))
are pairwise disjoint.
If α
is a linear succ order, β
is a preorder, and f : α → β
is a monotone function, then
the intervals set.Ico (f n) (f (order.succ n))
are pairwise disjoint.
If α
is a linear succ order, β
is a preorder, and f : α → β
is a monotone function, then
the intervals set.Ioo (f n) (f (order.succ n))
are pairwise disjoint.
If α
is a linear pred order, β
is a preorder, and f : α → β
is a monotone function, then
the intervals set.Ioc (f order.pred n) (f n)
are pairwise disjoint.
If α
is a linear pred order, β
is a preorder, and f : α → β
is a monotone function, then
the intervals set.Ico (f order.pred n) (f n)
are pairwise disjoint.
If α
is a linear pred order, β
is a preorder, and f : α → β
is a monotone function, then
the intervals set.Ioo (f order.pred n) (f n)
are pairwise disjoint.
If α
is a linear succ order, β
is a preorder, and f : α → β
is an antitone function, then
the intervals set.Ioc (f (order.succ n)) (f n)
are pairwise disjoint.
If α
is a linear succ order, β
is a preorder, and f : α → β
is an antitone function, then
the intervals set.Ico (f (order.succ n)) (f n)
are pairwise disjoint.
If α
is a linear succ order, β
is a preorder, and f : α → β
is an antitone function, then
the intervals set.Ioo (f (order.succ n)) (f n)
are pairwise disjoint.
If α
is a linear pred order, β
is a preorder, and f : α → β
is an antitone function, then
the intervals set.Ioc (f n) (f (order.pred n))
are pairwise disjoint.
If α
is a linear pred order, β
is a preorder, and f : α → β
is an antitone function, then
the intervals set.Ico (f n) (f (order.pred n))
are pairwise disjoint.
If α
is a linear pred order, β
is a preorder, and f : α → β
is an antitone function, then
the intervals set.Ioo (f n) (f (order.pred n))
are pairwise disjoint.