Zulip Chat Archive

Stream: mathlib4

Topic: Private lemmas on pointwise set ops appearing in simp?


Yakov Pechersky (Dec 29 2023 at 15:26):

MWE:

import Mathlib.Data.Set.Pointwise.Basic

example {α : Type*} [OrderedCommGroup α] {s : Set α} (h : BddBelow s) :
    BddAbove (s⁻¹) := by
  simp? -- Try this: simp only [_private.Mathlib.Data.Set.Pointwise.Basic.0.Set.involutiveInv._eq_1]
  sorry

Alex J. Best (Dec 29 2023 at 15:46):

I think this is the same lemma as https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/simp.20tracing.20suggests.20private.20simp.20theorems/near/406552591


Last updated: May 02 2025 at 03:31 UTC