Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2022-08-25 00:16 4b440bb0

View on Github →

refactor(order/well_founded_set): golf, review API (#11303)

New lemmas

About set.well_founded_on

  • set.well_founded_on.mono, set.well_founded_on.mono_set;
  • set.well_founded_on.union, set.well_founded_on_union, finset.well_founded_on, set.finite.well_founded_on, set.subsingleton.well_founded_on, set.well_founded_on_empty, set.well_founded_on_singleton, set.well_founded_on_insert, set.well_founded_on.insert;

About set.is_wf

  • set.is_wf_union;
  • set.finite.is_wf, finset.is_wf, set.is_wf_empty, set.is_wf_singleton, set.subsingleton.is_wf, set.is_wf_insert, set.is_wf.insert;
  • finset.is_wf_bUnion

About set.partially_well_ordered_on

  • set.partially_well_ordered_on.union, set.partially_well_ordered_on_union;
  • set.finite.partially_well_ordered_on, finset.partially_well_ordered_on, set.partially_well_ordered_on_empty, set.partially_well_ordered_on_singleton, set.partially_well_ordered_on_insert (an iff), set.partially_well_ordered_on.insert, set.subsingleton.partially_well_ordered_on;

About set.is_pwo

  • set.is_pwo.image_of_monotone_on, set.is_pwo_union;
  • finset.is_pwo, set.is_pwo_insert;
  • finset.is_pwo_bUnion;

Other API changes

  • Definitions lemmas now use ∀ n, f n ∈ s instead of range f ⊆ s.
  • Many lemmas now use weaker TC assumptions (e.g., preorder instead of partial_order).
  • set.is_wf_iff_no_descending_seq now uses (f : ℕ → α) (hf : strict_anti f) instead of f : order_dual ℕ ↪o α.
  • The order of binders in the hf argument of set.partially_well_ordered_on.image_of_monotone_on was changed to match monotone_on.
  • set.is_pwo.prod now allows sets from different types.
  • finset.is_wf_sup and finset.is_pwo_sup are now iffs

Estimated changes

deleted theorem finset.is_pwo
added theorem finset.is_pwo_bUnion
modified theorem finset.is_pwo_sup
deleted theorem finset.is_wf
added theorem finset.is_wf_bUnion
modified theorem finset.is_wf_sup
deleted theorem finset.well_founded_on
modified theorem pi.is_pwo
deleted theorem set.finite.is_pwo
deleted theorem set.fintype.is_pwo
deleted theorem set.is_pwo.insert
deleted theorem set.is_pwo.is_wf
modified theorem set.is_pwo.mono
deleted theorem set.is_pwo.mul
modified theorem set.is_pwo.prod
deleted theorem set.is_pwo.union
modified def set.is_pwo
modified theorem set.is_pwo_empty
added theorem set.is_pwo_insert
added theorem set.is_pwo_of_finite
modified theorem set.is_pwo_singleton
added theorem set.is_pwo_union
added theorem set.is_wf.insert
deleted theorem set.is_wf.is_pwo
modified theorem set.is_wf.le_min_iff
modified theorem set.is_wf.min_le
deleted theorem set.is_wf.min_mul
modified theorem set.is_wf.mono
deleted theorem set.is_wf.mul
deleted theorem set.is_wf.union
modified theorem set.is_wf_iff_is_pwo
added theorem set.is_wf_insert
added theorem set.is_wf_singleton
added theorem set.is_wf_union
modified def set.well_founded_on
modified theorem set.well_founded_on_iff
modified theorem well_founded.is_wf