Commit 2025-12-02 12:55 a2f9dca9

View on Github →

chore(Order/Basic): use @[to_dual] (#31903) This PR uses @[to_dual] in the rest of Mathlib.Order.Basic. I noticed that it was annoying to have to manually specify the reorder argument when it was very obvious what it should be, when using to_dual self. So, I created #31902 to do this automatically. Eq.trans_ge is not what the lemma name would make me think it is. So for now I've left it and similar lemmas without a tag, to avoid unnecessarily creating new lemmas. There are some lemmas like Function.Injective.linearOrder that have a hypothesis of the form ∀ {x y}, f x ≤ f y ↔ x ≤ y. In order to dualize this, we need to swap x and y, but it is not yet possible to reorder arguments of arguments.

Estimated changes

added theorem DenselyOrdered.dense'
deleted theorem PUnit.min_eq
modified theorem Prod.GCongr.mk_le_mk
modified theorem Prod.le_def
modified theorem Prod.mk_le_mk
deleted theorem Prod.mk_le_swap
deleted theorem Prod.mk_lt_swap
modified theorem Prod.swap_le_mk
modified theorem Prod.swap_le_swap
modified theorem Prod.swap_lt_mk
deleted theorem eq_of_forall_gt_iff
modified theorem exists_between
deleted theorem forall_gt_iff_le
deleted theorem le_of_forall_gt
deleted theorem max_rec'
deleted theorem max_rec
deleted theorem update_le_iff
deleted theorem update_le_self_iff
deleted theorem update_lt_self_iff