Zulip Chat Archive

Stream: new members

Topic: Proving an equality with supremum of an indexed family


Vlad (Apr 12 2024 at 21:51):

While the equation below appears straightforward, I'm wondering if there's a relevant lemma that could be helpful in proving it. I found lemmas about supremum of an (bounded) indexed family in the Real, Language, and Cardinality packages, but I haven't been able to connect them directly to this problem.

import Lean
import Mathlib.Tactic
open Lean Finset Algebra

example {i : } {xs: Array }
  (h0: 0 < i)
  (hi: i < xs.size)
  := calc xs[i] + ( a  range i, xs[a]'sorry)
        _ =  a  range i, (xs[i] + xs[a]'sorry)   := sorry -- by rw [add_ciSup]

Last updated: May 02 2025 at 03:31 UTC