@[class]
- le : α → α → Prop
- lt : α → α → Prop
- le_refl : ∀ (a : α), a ≤ a
- le_trans : ∀ (a b c_1 : α), a ≤ b → b ≤ c_1 → a ≤ c_1
- lt_iff_le_not_le : (∀ (a b : α), a < b ↔ a ≤ b ∧ ¬b ≤ a) . "order_laws_tac"
A preorder is a reflexive, transitive relation ≤
with a < b
defined in the obvious way.
Instances
- partial_order.to_preorder
- units.preorder
- add_units.preorder
- with_zero.preorder
- multiplicative.preorder
- additive.preorder
- directed_order.to_preorder
- order_dual.preorder
- pi.preorder
- subtype.preorder
- prod.preorder
- with_bot.preorder
- with_top.preorder
- rat.preorder
- associates.preorder
- finsupp.preorder
- cau_seq.preorder
- real.preorder
- bitvec.preorder
- filter.germ.preorder
- zsqrtd.preorder
- measure_theory.simple_func.preorder
- measure_theory.ae_eq_fun.preorder
- Preorder.preorder
- lex_preorder
- dlex_preorder
- onote.preorder
- nonote.preorder
- surreal.preorder
@[class]
- le : α → α → Prop
- lt : α → α → Prop
- le_refl : ∀ (a : α), a ≤ a
- le_trans : ∀ (a b c_1 : α), a ≤ b → b ≤ c_1 → a ≤ c_1
- lt_iff_le_not_le : (∀ (a b : α), a < b ↔ a ≤ b ∧ ¬b ≤ a) . "order_laws_tac"
- le_antisymm : ∀ (a b : α), a ≤ b → b ≤ a → a = b
A partial order is a reflexive, transitive, antisymmetric relation ≤
.
Instances
- linear_order.to_partial_order
- semilattice_sup.to_partial_order
- semilattice_inf.to_partial_order
- order_top.to_partial_order
- order_bot.to_partial_order
- ordered_comm_monoid.to_partial_order
- ordered_add_comm_monoid.to_partial_order
- units.partial_order
- add_units.partial_order
- with_zero.partial_order
- ordered_cancel_add_comm_monoid.to_partial_order
- ordered_cancel_comm_monoid.to_partial_order
- ordered_add_comm_group.to_partial_order
- ordered_comm_group.to_partial_order
- multiplicative.partial_order
- additive.partial_order
- order_dual.partial_order
- pi.partial_order
- subtype.partial_order
- prod.partial_order
- with_bot.partial_order
- with_top.partial_order
- multiset.partial_order
- finset.partial_order
- rat.partial_order
- associates.partial_order
- submonoid.partial_order
- add_submonoid.partial_order
- subgroup.partial_order
- add_subgroup.partial_order
- finsupp.partial_order
- submodule.partial_order
- setoid.partial_order
- con.partial_order
- add_con.partial_order
- subsemiring.partial_order
- subalgebra.partial_order
- ordinal.partial_order
- enat.partial_order
- pequiv.partial_order
- filter.partial_order
- topological_space.partial_order
- topological_space.opens.partial_order
- real.partial_order
- uniform_space.partial_order
- enorm.partial_order
- semiquot.partial_order
- filter.germ.partial_order
- setoid.partition.partial_order
- structure_groupoid.partial_order
- measurable_space.partial_order
- measurable_space.dynkin_system.partial_order
- measure_theory.measure.partial_order
- measure_theory.simple_func.partial_order
- measure_theory.ae_eq_fun.partial_order
- PartialOrder.partial_order
- lex_partial_order
- dlex_partial_order
- pilex.partial_order
- ring.fractional_ideal.partial_order
- surreal.partial_order
- open_subgroup.partial_order
- open_add_subgroup.partial_order
@[class]
- le : α → α → Prop
- lt : α → α → Prop
- le_refl : ∀ (a : α), a ≤ a
- le_trans : ∀ (a b c_1 : α), a ≤ b → b ≤ c_1 → a ≤ c_1
- lt_iff_le_not_le : (∀ (a b : α), a < b ↔ a ≤ b ∧ ¬b ≤ a) . "order_laws_tac"
- le_antisymm : ∀ (a b : α), a ≤ b → b ≤ a → a = b
- le_total : ∀ (a b : α), a ≤ b ∨ b ≤ a
A linear order is reflexive, transitive, antisymmetric and total relation ≤
.
Instances
- decidable_linear_order.to_linear_order
- units.linear_order
- add_units.linear_order
- with_zero.linear_order
- multiplicative.linear_order
- additive.linear_order
- linear_ordered_semiring.to_linear_order
- linear_ordered_ring.to_linear_order
- linear_nonneg_ring.to_linear_order
- linear_ordered_comm_group_with_zero.to_linear_order
- nat.linear_order
- order_dual.linear_order
- subtype.linear_order
- with_bot.linear_order
- with_top.linear_order
- list.linear_order
- fin.linear_order
- rat.linear_order
- cardinal.linear_order
- real.linear_order
- ereal.linear_order
- LinearOrder.linear_order
- lex_linear_order
- dlex_linear_order
- nonote.linear_order
- surreal.linear_order
@[instance]
@[instance]
Equations
- decidable_lt_of_decidable_le a b = dite (a ≤ b) (λ (hab : a ≤ b), dite (b ≤ a) (λ (hba : b ≤ a), decidable.is_false _) (λ (hba : ¬b ≤ a), decidable.is_true _)) (λ (hab : ¬a ≤ b), decidable.is_false _)
@[instance]
Equations
- decidable_eq_of_decidable_le a b = dite (a ≤ b) (λ (hab : a ≤ b), dite (b ≤ a) (λ (hba : b ≤ a), decidable.is_true _) (λ (hba : ¬b ≤ a), decidable.is_false _)) (λ (hab : ¬a ≤ b), decidable.is_false _)
@[instance]
@[class]
- le : α → α → Prop
- lt : α → α → Prop
- le_refl : ∀ (a : α), a ≤ a
- le_trans : ∀ (a b c_1 : α), a ≤ b → b ≤ c_1 → a ≤ c_1
- lt_iff_le_not_le : (∀ (a b : α), a < b ↔ a ≤ b ∧ ¬b ≤ a) . "order_laws_tac"
- le_antisymm : ∀ (a b : α), a ≤ b → b ≤ a → a = b
- le_total : ∀ (a b : α), a ≤ b ∨ b ≤ a
- decidable_le : decidable_rel has_le.le
- decidable_eq : decidable_eq α
- decidable_lt : decidable_rel has_lt.lt
Instances
- units.decidable_linear_order
- add_units.decidable_linear_order
- with_zero.decidable_linear_order
- canonically_linear_ordered_add_monoid.to_decidable_linear_order
- decidable_linear_ordered_cancel_add_comm_monoid.to_decidable_linear_order
- decidable_linear_ordered_add_comm_group.to_decidable_linear_order
- multiplicative.decidable_linear_order
- additive.decidable_linear_order
- decidable_linear_ordered_semiring.to_decidable_linear_order
- complete_linear_order.to_decidable_linear_order
- conditionally_complete_linear_order.to_decidable_linear_order
- conditionally_complete_linear_order_bot.to_decidable_linear_order
- nonempty_fin_lin_ord.to_decidable_linear_order
- nat.decidable_linear_order
- int.decidable_linear_order
- bool.decidable_linear_order
- order_dual.decidable_linear_order
- subtype.decidable_linear_order
- with_bot.decidable_linear_order
- with_top.decidable_linear_order
- list.decidable_linear_order
- fin.decidable_linear_order
- pnat.decidable_linear_order
- rat.decidable_linear_order
- char.decidable_linear_order
- string.decidable_linear_order
- cardinal.decidable_linear_order
- ordinal.decidable_linear_order
- enat.decidable_linear_order
- real.decidable_linear_order
- nnreal.decidable_linear_order
- pos_num.decidable_linear_order
- znum.decidable_linear_order
- zsqrtd.decidable_linear_order
- lex_decidable_linear_order
- dlex_decidable_linear_order
- nonote.decidable_linear_order
@[instance]
Equations
@[instance]
Equations
@[instance]
Equations
@[instance]
Equations
@[instance]