Zulip Chat Archive

Stream: general

Topic: Apply? suggests refines giving diff goals but just intros


Arav Bhattacharyya (Mar 06 2025 at 20:39):

Hi! I have this code where I forgot to intro a hypothesis and ran apply?. It suggests refine fun h => ?h many times, each time giving a different set of goals (this actually just gives the same as intro h). I think this is a bug as it should not give different goals for the same suggestion. I believe it is just suggesting things for after intro h

import Mathlib.MeasureTheory.Measure.LevyProkhorovMetric

open Topology Metric Filter Set ENNReal NNReal ProbabilityMeasure TopologicalSpace

namespace MeasureTheory


variable {Ω : Type*} [MeasurableSpace Ω] [PseudoMetricSpace Ω] [SeparableSpace Ω]
[OpensMeasurableSpace Ω]
variable {μ :   Set Ω  }


variable (S : Set (ProbabilityMeasure Ω))


lemma claim5point2 (U :   Set Ω) (O :  i, IsOpen (U i))
    (hcomp: IsCompact (closure S)) (ε : 0) :
     (k : ),  μ  S, μ ( (i  k), U i) > 1 - ε := by
  by_contra! nh
  choose μ  hμε using nh

  obtain μnew, hμtwo, sub, tub, bub := hcomp.isSeqCompact (fun n =>  subset_closure <|  n)
  have thing n := calc
    μnew ( (i  n), U i)
    _  liminf (fun k => μ (sub k) ( (i  n), U i)) atTop := by
      sorry
    _  liminf (fun k => μ (sub k) ( (i  k), U i)) atTop := by
      sorry
    _  1 - ε := by
      apply Filter.liminf_le_of_le
      · sorry
      · simp only [eventually_atTop, ge_iff_le, forall_exists_index]
        intros b c
        apply?
  sorry

Last updated: May 02 2025 at 03:31 UTC