Zulip Chat Archive

Stream: lean4

Topic: Some syntaх question


YurySerdyuk (Apr 21 2025 at 13:01):

Hi !
I would like to prove a property with some specific name P for a set S.
Formally , I would like to write something like this:

lemma name ( S : set type ) ( h : hypothesis about S ) : P S := by ...

But the Lean gives the message for such record :
function expected at
P
term has type
?m.62

What is wrong with my notation ?

Ruben Van de Velde (Apr 21 2025 at 13:09):

What does P mean?

YurySerdyuk (Apr 21 2025 at 13:09):

Some name

Ruben Van de Velde (Apr 21 2025 at 13:25):

Please share a #mwe, we can't help you with such vague questions

YurySerdyuk (Apr 21 2025 at 13:28):

More concretely I would like to prove that the specific collection of sets is a topology :

lemma openness (T : Set (Set )) (h : T = {O : Set  | O =    a  O,  b > 0, Set.range (fun n :  => a + n * b)  O}) :
  IsTopology T := by
  rw [h]
  refine' by simp, _⟩

What is wrong with my syntax ?

Ruben Van de Velde (Apr 21 2025 at 13:41):

Missing imports, for a start

YurySerdyuk (Apr 21 2025 at 13:43):

import Mathlib.Data.Set.Basic

lemma openness (T : Set (Set )) (h : T = {O : Set  | O =    a  O,  b > 0, Set.range (fun n :  => a + n * b)  O}) :
  IsTopology T := by
  rw [h]
  refine' by simp, _⟩
  -- Prove that the entire space ℤ is open.
  refine' by simp [Set.eq_univ_of_forall], _⟩

Ruben Van de Velde (Apr 21 2025 at 13:46):

Thanks. The issue is that IsTopology does not exist. Why did you think it would?

Ruben Van de Velde (Apr 21 2025 at 13:49):

That's a genuine question - how did you get to the point of writing IsTopology?

YurySerdyuk (Apr 21 2025 at 13:50):

I would like that isTopology would be the conjunction of the 4 corresponding properties. How to restructure the syntax of my proof ?

Kevin Buzzard (Apr 21 2025 at 13:55):

Is this code written by an LLM? Did you try reading a book on Lean?

Ruben Van de Velde (Apr 21 2025 at 13:55):

The first step if to define IsTopology, since it doesn't exist yet.

Ruben Van de Velde (Apr 21 2025 at 13:56):

But you still haven't answered my question why you wrote IsTopology in the first place


Last updated: May 02 2025 at 03:31 UTC