Zulip Chat Archive

Stream: Is there code for X?

Topic: variant of sSup_apply with sSup on both sides


Ira Fesefeldt (Jun 04 2024 at 07:29):

I am looking for something like sSup_apply for the complete Lattice of the pi type but that yields me again an sSup instead of an iSup. So, something like this:

import Mathlib.Data.Real.EReal

def my_type :=   EReal

noncomputable instance : CompleteLattice my_type := Pi.instCompleteLattice

theorem my_sSup_apply {α : Type} {f : α  my_type } {n : } :
    sSup { x |  y, f y = x} n = sSup { x |  y, f y n = x} := by
  sorry

Is there something like this? I only found sSup_apply, but I don't know how to make this iSup again into an sSup.

Eric Wieser (Jun 04 2024 at 11:54):

This works:

import Mathlib.Data.Real.EReal

abbrev my_type :=   EReal

theorem my_sSup_apply {α : Type} {f : α  my_type } {n : } :
    sSup { x |  y, f y = x} n = sSup { x |  y, f y n = x} := by
  rw [sSup_apply, iSup, Set.range]
  simp

Last updated: May 02 2025 at 03:31 UTC