Skip to content

Commit

Permalink
Merge remote-tracking branch 'origin/master' into test/add_remove_mer…
Browse files Browse the repository at this point in the history
…ge_conflict_label_in_ci
  • Loading branch information
adomani committed Jan 22, 2025
2 parents 96f6113 + 2cb1216 commit b60df39
Show file tree
Hide file tree
Showing 2 changed files with 11 additions and 5 deletions.
11 changes: 9 additions & 2 deletions Mathlib/Order/WellFoundedSet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -505,9 +505,13 @@ protected theorem IsWF.isPWO (hs : s.IsWF) : s.IsPWO := by
simp only [forall_mem_range, not_lt] at hm
exact ⟨m, m + 1, by omega, hm _⟩

/-- In a linear order, the predicates `Set.IsWF` and `Set.IsPWO` are equivalent. -/
/-- In a linear order, the predicates `Set.IsPWO` and `Set.IsWF` are equivalent. -/
theorem isPWO_iff_isWF : s.IsPWO ↔ s.IsWF :=
⟨IsPWO.isWF, IsWF.isPWO⟩

@[deprecated isPWO_iff_isWF (since := "2025-01-21")]
theorem isWF_iff_isPWO : s.IsWF ↔ s.IsPWO :=
⟨IsWF.isPWO, IsPWO.isWF⟩
isPWO_iff_isWF.symm

/--
If `α` is a linear order with well-founded `<`, then any set in it is a partially well-ordered set.
Expand Down Expand Up @@ -668,6 +672,9 @@ theorem BddBelow.wellFoundedOn_lt : BddBelow s → s.WellFoundedOn (· < ·) :=
theorem BddAbove.wellFoundedOn_gt : BddAbove s → s.WellFoundedOn (· > ·) :=
fun h => h.dual.wellFoundedOn_lt

theorem BddBelow.isWF : BddBelow s → IsWF s :=
BddBelow.wellFoundedOn_lt

end LocallyFiniteOrder

namespace Set.PartiallyWellOrderedOn
Expand Down
5 changes: 2 additions & 3 deletions Mathlib/RingTheory/HahnSeries/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -476,10 +476,9 @@ theorem BddBelow_zero [Nonempty Γ] : BddBelow (Function.support (0 : Γ → R))

variable [LocallyFiniteOrder Γ]

theorem suppBddBelow_supp_PWO (f : Γ → R)
(hf : BddBelow (Function.support f)) :
theorem suppBddBelow_supp_PWO (f : Γ → R) (hf : BddBelow (Function.support f)) :
(Function.support f).IsPWO :=
Set.isWF_iff_isPWO.mp hf.wellFoundedOn_lt
hf.isWF.isPWO

/-- Construct a Hahn series from any function whose support is bounded below. -/
@[simps]
Expand Down

0 comments on commit b60df39

Please sign in to comment.