Zulip Chat Archive

Stream: mathlib4

Topic: propose on a product space


Floris van Doorn (Apr 28 2023 at 14:49):

In the following code, the first example doesn't give any suggestions, while the second example gives some useful suggestions.

import Mathlib.Topology.SubsetProperties
import Mathlib.Tactic.Propose

example [TopologicalSpace X] [CompactSpace X] (K : Set (X × X)) (hK : IsClosed K) : False := by
  propose using hK -- no suggestions

example [TopologicalSpace X] [CompactSpace X] (K : Set X) (hK : IsClosed K) : False := by
  propose using hK -- multiple suggestions

Last updated: Dec 20 2023 at 11:08 UTC