Zulip Chat Archive

Stream: general

Topic: well_founded typeclass


Yaël Dillies (Dec 28 2021 at 18:17):

Consider

/-- The order on `ι →₀ ℕ` is well-founded. -/
lemma lt_wf : well_founded (@has_lt.lt (ι →₀ ) _) :=
subrelation.wf (sum_id_lt_of_lt) $ inv_image.wf _ nat.lt_wf

in file#data/finsupp/order. This could be generalized to ι →₀ α where α is well-founded itself. Do we want to handled well-foundedness with typeclasses?


Last updated: Dec 20 2023 at 11:08 UTC