leanprover-community / lean4game

Server to host lean games.
https://adam.math.hhu.de
GNU General Public License v3.0
197 stars 35 forks source link

Can't write "use (succ(succ a))" #258

Closed VasiliPupkin256 closed 2 months ago

VasiliPupkin256 commented 2 months ago

Goal: y ≤ y + succ (succ a)

I've had to go the long way use (a+2) rw [two_eq_succ_one] rw [one_eq_succ_zero] repeat rw [add_succ] rw [add_zero] rfl

Instead of just typing use (succ(succ a)) which is not allowed. PS: one can type use (succ a) though.

joneugster commented 2 months ago

I need some context :) Which game/level were you playing, NNG?

Is it more than just adding a space between succ and (, i.e. succ ( instead of succ(?

VasiliPupkin256 commented 2 months ago

It was Level 8 Inequality World. Yes, adding a space solved the issue. The parser is odd.

joneugster commented 2 months ago

Yes Im afraid this might be just how Lean works: its oddly whitespace sensitive although it gives the impression its not.