Zulip Chat Archive

Stream: Is there code for X?

Topic: supr over units ℤ


Eric Wieser (Sep 30 2021 at 12:41):

Do we have this anywhere?

lemma supr_units_int {α : Type*} (f : units   α) [complete_lattice α] :
   i : units ,  f i = f 1  f (-1) :=
sorry

docs#supr_bool_eq is close, but I'm not sure of the easiest way to glue it

Johan Commelin (Sep 30 2021 at 12:44):

Shouldn't there be general machinery for fintypes that folds over finset.univ or something like that?

Johan Commelin (Sep 30 2021 at 12:45):

Doing this just for units ℤ seems too specific. If I take the sup indexed by fin 5, I want 3 well-chosen simp/rw lemmas to turn it into

f 0  f 1  f 2  f 3  f 4

etc...

Anne Baanen (Sep 30 2021 at 12:45):

I know there's something along the lines of docs#int.units_eq_one_or, (EDIT:) and we have docs#units_int.univ

Eric Wieser (Sep 30 2021 at 12:46):

Converting to finset.sup sounds like the way to go

Eric Wieser (Sep 30 2021 at 12:46):

docs#finset.sup_eq_supr?

Yaël Dillies (Sep 30 2021 at 12:47):

Yup

Anne Baanen (Sep 30 2021 at 12:47):

And then perhaps docs#finset.sup_insert?


Last updated: Dec 20 2023 at 11:08 UTC