Zulip Chat Archive

Stream: new members

Topic: Problem of closed set


haotian liu (Mar 03 2024 at 06:19):

Is there a relevant theorem inside mathilb that accomplishes the proof of the following theorem? If not, is there a theorem that I can learn from?

have hdef_r_close {zset_r : Set } (hdef1 : zset_r = {x | (αleft  x  x  αright)}) : IsClosed (zset_r) := by
      sorry

Kyle Miller (Mar 03 2024 at 06:33):

Yes, docs#isClosed_Icc

haotian liu (Mar 03 2024 at 07:28):

Thank you very much!
Actually, I want to prove the following problem:

private theorem Is_closed_zset {αleft αright : } {g :   } {zset : Set }
    (hdef : zset = {x | (αleft  x  x  αright)  g x = 0}) (hg : Continuous g) :
    IsClosed (zset) := by
    sorry

Now, I can prove that zset_r = {x | (αleft ≤ x ∧ x ≤ αright)} is closed.
Is there any theorem that proves that a subset of a closed set is also a closed set?
Or is there any theorem that proves that the set of zeros of a continuous function is a closed set?

Kyle Miller (Mar 03 2024 at 07:32):

theorem Is_closed_zset {αleft αright : } {g :   } {zset : Set }
    (hdef : zset = {x | (αleft  x  x  αright)  g x = 0}) (hg : Continuous g) :
    IsClosed zset := by
  subst zset
  apply IsClosed.inter
  · exact isClosed_Icc
  · change IsClosed (g ⁻¹' {0})
    apply IsClosed.preimage hg
    exact T1Space.t1 0

haotian liu (Mar 03 2024 at 07:41):

Thank you very much!


Last updated: May 02 2025 at 03:31 UTC