Documentation

Mathlib.Order.PropInstances

The order on Prop #

Instances on Prop such as DistribLattice, BoundedOrder, LinearOrder.

Propositions form a bounded order.

Equations
instance Prop.le_isTotal :
IsTotal Prop fun (x x_1 : Prop) => x x_1
Equations
@[simp]
theorem sup_Prop_eq :
(fun (x x_1 : Prop) => x x_1) = fun (x x_1 : Prop) => x x_1
@[simp]
theorem inf_Prop_eq :
(fun (x x_1 : Prop) => x x_1) = fun (x x_1 : Prop) => x x_1
theorem Pi.disjoint_iff {ι : Type u_1} {α' : ιType u_2} [(i : ι) → PartialOrder (α' i)] [(i : ι) → OrderBot (α' i)] {f : (i : ι) → α' i} {g : (i : ι) → α' i} :
Disjoint f g ∀ (i : ι), Disjoint (f i) (g i)
theorem Pi.codisjoint_iff {ι : Type u_1} {α' : ιType u_2} [(i : ι) → PartialOrder (α' i)] [(i : ι) → OrderTop (α' i)] {f : (i : ι) → α' i} {g : (i : ι) → α' i} :
Codisjoint f g ∀ (i : ι), Codisjoint (f i) (g i)
theorem Pi.isCompl_iff {ι : Type u_1} {α' : ιType u_2} [(i : ι) → PartialOrder (α' i)] [(i : ι) → BoundedOrder (α' i)] {f : (i : ι) → α' i} {g : (i : ι) → α' i} :
IsCompl f g ∀ (i : ι), IsCompl (f i) (g i)
@[simp]
theorem Prop.disjoint_iff {P : Prop} {Q : Prop} :
Disjoint P Q ¬(P Q)
@[simp]
theorem Prop.codisjoint_iff {P : Prop} {Q : Prop} :
@[simp]
theorem Prop.isCompl_iff {P : Prop} {Q : Prop} :
IsCompl P Q ¬(P Q)