Zulip Chat Archive

Stream: new members

Topic: worth copying defeq uIoc/uIcc lemmas?


llllvvuu (Feb 09 2024 at 00:50):

import Mathlib.Data.Set.Intervals.UnorderedInterval

example {E : Type*} [LinearOrder E] {a b : E} : Set.uIoc a b  Set.uIcc a b := by
  -- exact? fails
  -- simp made no progress
  -- apply? returns junk
  exact Set.Ioc_subset_Icc_self -- succeeds

Should a copy of the Ioc/Icc API exist for uIoc/uIcc?

Eric Wieser (Feb 09 2024 at 07:00):

Yes, I think it should

Eric Wieser (Feb 09 2024 at 07:00):

I'm surprised that proof works

Eric Wieser (Feb 09 2024 at 07:02):

Either that, or we should make the u variants abbrevs

Eric Wieser (Feb 09 2024 at 07:02):

Maybe @Yaël Dillies has an opinion?

Yaël Dillies (Feb 09 2024 at 08:36):

My two (overly informed) cents:

  • They should be abbrev on the basis that we use them relatively little and that there are many lemmas to copy
  • They should not be abbrev for performance because a and b appear twice in their definition (uIcc a b = Icc (a ⊓ b) (a ⊔ b)

Last updated: May 02 2025 at 03:31 UTC