Documentation

Mathlib.Order.UpperLower.Relative

Properties of relative upper/lower sets #

This file proves results on IsRelUpperSet and IsRelLowerSet.

theorem IsRelUpperSet.prop_of_mem {α : Type u_1} {s : Set α} {a : α} {P : αProp} [LE α] (hs : IsRelUpperSet s P) (h : a s) :
P a
theorem IsRelLowerSet.prop_of_mem {α : Type u_1} {s : Set α} {a : α} {P : αProp} [LE α] (hs : IsRelLowerSet s P) (h : a s) :
P a
@[simp]
theorem isRelUpperSet_empty {α : Type u_1} {P : αProp} [LE α] :
@[simp]
theorem isRelLowerSet_empty {α : Type u_1} {P : αProp} [LE α] :
@[simp]
theorem isRelUpperSet_self {α : Type u_1} {s : Set α} [LE α] :
IsRelUpperSet s fun (x : α) => x s
@[simp]
theorem isRelLowerSet_self {α : Type u_1} {s : Set α} [LE α] :
IsRelLowerSet s fun (x : α) => x s
theorem IsRelUpperSet.union {α : Type u_1} {s t : Set α} {P : αProp} [LE α] (hs : IsRelUpperSet s P) (ht : IsRelUpperSet t P) :
theorem IsRelLowerSet.union {α : Type u_1} {s t : Set α} {P : αProp} [LE α] (hs : IsRelLowerSet s P) (ht : IsRelLowerSet t P) :
theorem IsRelUpperSet.inter {α : Type u_1} {s t : Set α} {P : αProp} [LE α] (hs : IsRelUpperSet s P) (ht : IsRelUpperSet t P) :
theorem IsRelLowerSet.inter {α : Type u_1} {s t : Set α} {P : αProp} [LE α] (hs : IsRelLowerSet s P) (ht : IsRelLowerSet t P) :
theorem IsRelUpperSet.sUnion {α : Type u_1} {P : αProp} [LE α] {S : Set (Set α)} (hS : sS, IsRelUpperSet s P) :
theorem IsRelLowerSet.sUnion {α : Type u_1} {P : αProp} [LE α] {S : Set (Set α)} (hS : sS, IsRelLowerSet s P) :
theorem IsRelUpperSet.iUnion {α : Type u_1} {ι : Sort u_2} {P : αProp} [LE α] {f : ιSet α} (hf : ∀ (i : ι), IsRelUpperSet (f i) P) :
IsRelUpperSet (⋃ (i : ι), f i) P
theorem IsRelLowerSet.iUnion {α : Type u_1} {ι : Sort u_2} {P : αProp} [LE α] {f : ιSet α} (hf : ∀ (i : ι), IsRelLowerSet (f i) P) :
IsRelLowerSet (⋃ (i : ι), f i) P
theorem IsRelUpperSet.iUnion₂ {α : Type u_1} {ι : Sort u_2} {κ : ιSort u_3} {P : αProp} [LE α] {f : (i : ι) → κ iSet α} (hf : ∀ (i : ι) (j : κ i), IsRelUpperSet (f i j) P) :
IsRelUpperSet (⋃ (i : ι), ⋃ (j : κ i), f i j) P
theorem IsRelLowerSet.iUnion₂ {α : Type u_1} {ι : Sort u_2} {κ : ιSort u_3} {P : αProp} [LE α] {f : (i : ι) → κ iSet α} (hf : ∀ (i : ι) (j : κ i), IsRelLowerSet (f i j) P) :
IsRelLowerSet (⋃ (i : ι), ⋃ (j : κ i), f i j) P
theorem IsRelUpperSet.sInter {α : Type u_1} {P : αProp} [LE α] {S : Set (Set α)} (hS : S.Nonempty) (hf : sS, IsRelUpperSet s P) :
theorem IsRelLowerSet.sInter {α : Type u_1} {P : αProp} [LE α] {S : Set (Set α)} (hS : S.Nonempty) (hf : sS, IsRelLowerSet s P) :
theorem IsRelUpperSet.iInter {α : Type u_1} {ι : Sort u_2} {P : αProp} [LE α] [Nonempty ι] {f : ιSet α} (hf : ∀ (i : ι), IsRelUpperSet (f i) P) :
IsRelUpperSet (⋂ (i : ι), f i) P
theorem IsRelLowerSet.iInter {α : Type u_1} {ι : Sort u_2} {P : αProp} [LE α] [Nonempty ι] {f : ιSet α} (hf : ∀ (i : ι), IsRelLowerSet (f i) P) :
IsRelLowerSet (⋂ (i : ι), f i) P
theorem IsRelUpperSet.iInter₂ {α : Type u_1} {ι : Sort u_2} {κ : ιSort u_3} {P : αProp} [LE α] [Nonempty ι] [∀ (i : ι), Nonempty (κ i)] {f : (i : ι) → κ iSet α} (hf : ∀ (i : ι) (j : κ i), IsRelUpperSet (f i j) P) :
IsRelUpperSet (⋂ (i : ι), ⋂ (j : κ i), f i j) P
theorem IsRelLowerSet.iInter₂ {α : Type u_1} {ι : Sort u_2} {κ : ιSort u_3} {P : αProp} [LE α] [Nonempty ι] [∀ (i : ι), Nonempty (κ i)] {f : (i : ι) → κ iSet α} (hf : ∀ (i : ι) (j : κ i), IsRelLowerSet (f i j) P) :
IsRelLowerSet (⋂ (i : ι), ⋂ (j : κ i), f i j) P
theorem isUpperSet_subtype_iff_isRelUpperSet {α : Type u_1} {P : αProp} [LE α] {s : Set { x : α // P x }} :
theorem isLowerSet_subtype_iff_isRelLowerSet {α : Type u_1} {P : αProp} [LE α] {s : Set { x : α // P x }} :
instance instSetLikeRelUpperSet {α : Type u_1} {P : αProp} [LE α] :
Equations
instance instSetLikeRelLowerSet {α : Type u_1} {P : αProp} [LE α] :
Equations
theorem RelUpperSet.isRelUpperSet {α : Type u_1} {P : αProp} [LE α] (u : RelUpperSet P) :
IsRelUpperSet (↑u) P
theorem RelLowerSet.isRelLowerSet {α : Type u_1} {P : αProp} [LE α] (l : RelLowerSet P) :
IsRelLowerSet (↑l) P
theorem isRelUpperSet_Icc_le {α : Type u_1} {a : α} [Preorder α] {c : α} :
IsRelUpperSet (Set.Icc a c) fun (x : α) => x c
theorem isRelLowerSet_Icc_ge {α : Type u_1} {a : α} [Preorder α] {c : α} :
IsRelLowerSet (Set.Icc c a) fun (x : α) => c x