Zulip Chat Archive

Stream: lean4

Topic: parsing error for `set_option` after docstring comment


Arien Malec (Feb 04 2023 at 22:37):

#mwe

-- /-- multiline
-- comment-/ -- if you uncomment this, syntax error
set_option linter.deprecated false in
theorem bar {α β: Type _}: α = β := sorry

-- this position is OK
--set_option linter.deprecated false in
/-- multiline
comment-/
set_option linter.deprecated false in -- syntax error
def foo {α :Type _} : α -> α := sorry

Mario Carneiro (Feb 04 2023 at 22:38):

yes this is expected behavior

Reid Barton (Feb 04 2023 at 23:00):

That's a docstring, not (just) a multiline comment, since it starts with /--

Reid Barton (Feb 04 2023 at 23:00):

/- this is a
multiline comment -/

Last updated: Dec 20 2023 at 11:08 UTC