This theory is a continuation of Order_ZF and talks about maximum and minimum of a set, supremum and infimum and strict (not reflexive) versions of order relations.
In this section we show that maximum and minimum are unique if they exist. We also show that union of sets that have maxima (minima) has a maximum (minimum). We also show that singletons have maximum and minimum. All this allows to show (in Finite_ZF) that every finite set has well-defined maximum and minimum.
A somewhat technical fact that allows to reduce the number of premises in some theorems: the assumption that a set has a maximum implies that it is not empty.
lemma set_max_not_empty:
assumes
If a set has a maximum implies that it is not empty.
lemma set_min_not_empty:
assumes
If a set has a supremum then it cannot be empty. We are probably using the fact that
lemma set_sup_not_empty:
assumes
If a set has an infimum then it cannot be empty.
lemma set_inf_not_empty:
assumes
For antisymmetric relations maximum of a set is unique if it exists.
lemma Order_ZF_4_L1:
assumes A1:
For antisymmetric relations minimum of a set is unique if it exists.
lemma Order_ZF_4_L2:
assumes A1:
Maximum of a set has desired properties.
lemma Order_ZF_4_L3:
assumes A1:
Minimum of a set has desired properties.
lemma Order_ZF_4_L4:
assumes A1:
For total and transitive relations a union a of two sets that have maxima has a maximum.
lemma Order_ZF_4_L5:
assumes A1:
For total and transitive relations A union a of two sets that have minima has a minimum.
lemma Order_ZF_4_L6:
assumes A1:
Set that has a maximum is bounded above.
lemma Order_ZF_4_L7:
assumes
Set that has a minimum is bounded below.
lemma Order_ZF_4_L8A:
assumes
A subset of a set that has a maximum is bounded above.
lemma max_subset_bounded:
assumes
A subset of a set that has a minimum is bounded below.
lemma min_subset_bounded:
assumes
For reflexive relations singletons have a minimum and maximum.
lemma Order_ZF_4_L8:
assumes
For total and transitive relations if we add an element to a set that has a maximum, the set still has a maximum.
lemma Order_ZF_4_L9:
assumes A1:
For total and transitive relations if we add an element to a set that has a minimum, the set still has a minimum.
lemma Order_ZF_4_L10:
assumes A1:
If the order relation has a property that every nonempty bounded set attains a minimum (for example integers are like that), then every nonempty set bounded below attains a minimum.
lemma Order_ZF_4_L11:
assumes A1:
A dual to Order_ZF_4_L11: If the order relation has a property that every nonempty bounded set attains a maximum (for example integers are like that), then every nonempty set bounded above attains a maximum.
lemma Order_ZF_4_L11A:
assumes A1:
If a set has a minimum and
lemma Order_ZF_4_L12:
assumes
If a set has a maximum and all its elements are less or equal than
lemma Order_ZF_4_L13:
assumes
If an element belongs to a set and is greater or equal than all elements of that set, then it is the maximum of that set.
lemma Order_ZF_4_L14:
assumes A1:
If an element belongs to a set and is less or equal than all elements of that set, then it is the minimum of that set.
lemma Order_ZF_4_L15:
assumes A1:
If a set does not have a maximum, then for any its element we can find one that is (strictly) greater.
lemma Order_ZF_4_L16:
assumes A1:
In this section we consider the notions of supremum and infimum a set.
Elements of the set of upper bounds are indeed upper bounds. Isabelle also thinks it is obvious.
lemma Order_ZF_5_L1:
assumes
Elements of the set of lower bounds are indeed lower bounds. Isabelle also thinks it is obvious.
lemma Order_ZF_5_L2:
assumes
If the set of upper bounds has a minimum, then the supremum
is less or equal than any upper bound. We can probably do away with
the assumption that
lemma Order_ZF_5_L3:
assumes A1:
Supremum is less or equal than any upper bound.
lemma sup_leq_up_bnd:
assumes
Infimum is greater or equal than any lower bound. This lemma is obsolete and will be removed. Use inf_geq_lo_bnd instead.
lemma Order_ZF_5_L4:
assumes A1:
Infimum is greater or equal than any upper bound.
lemma inf_geq_lo_bnd:
assumes
If
lemma Order_ZF_5_L5:
assumes A1:
The dual theorem to Order_ZF_5_L5: if
lemma inf_glb:
assumes
Supremum and infimum of a singleton is the element.
lemma sup_inf_singl:
assumes
If a set has a maximum, then the maximum is the supremum. This lemma is obsolete, use max_is_sup instead.
lemma Order_ZF_5_L6:
assumes A1:
Another version of Order_ZF_5_L6 that: if a sat has a maximum then it has a supremum and the maximum is the supremum.
lemma max_is_sup:
assumes
Minimum is the infimum if it exists.
lemma min_is_inf:
assumes
For reflexive and total relations two-element set has a minimum and a maximum.
lemma min_max_two_el:
assumes
For antisymmetric, reflexive and total relations two-element set has a supremum and infimum.
lemma inf_sup_two_el:
assumes
A sufficient condition for the supremum to be in the space.
lemma sup_in_space:
assumes
A sufficient condition for the infimum to be in the space.
lemma inf_in_space:
assumes
Properties of supremum of a set for complete relations.
lemma Order_ZF_5_L7:
assumes A1:
Infimum of the set of infima of a collection of sets is infimum of the union.
lemma inf_inf:
assumes
Supremum of the set of suprema of a collection of sets is supremum of the union.
lemma sup_sup:
assumes
If the relation is a linear order then for any
element
lemma Order_ZF_5_L8:
assumes A1:
One of the problems with translating formalized mathematics from
Metamath to IsarMathLib is that Metamath uses strict orders (of the
We define a strict version of a relation by removing the
definition
A reformulation of the definition of a strict version of an order.
lemma def_of_strict_ver:
showsThe next lemma is about the strict version of an antisymmetric relation.
lemma strict_of_antisym:
assumes A1:
The strict version of totality.
lemma strict_of_tot:
assumes
A trichotomy law for the strict version of a total and antisymmetric relation. It is kind of interesting that one does not need the full linear order for this.
lemma strict_ans_tot_trich:
assumes A1:
A trichotomy law for linear order. This is a special case of strict_ans_tot_trich.
corollary strict_lin_trich:
assumes A1:
For an antisymmetric relation if a pair is in relation then the reversed pair is not in the strict version of the relation.
lemma geq_impl_not_less:
assumes A1:
If an antisymmetric relation is transitive, then the strict version is also transitive, an explicit version strict_of_transB below.
lemma strict_of_transA:
assumes A1:
If an antisymmetric relation is transitive, then the strict version is also transitive.
lemma strict_of_transB:
assumes A1:
The next lemma provides a condition that is satisfied by the strict version of a relation if the original relation is a complete linear order.
lemma strict_of_compl:
assumes A1:
Strict version of a relation on a set is a relation on that set.
lemma strict_ver_rel:
assumes A1: