Zulip Chat Archive
Stream: lean4
Topic: Mysterious error message
Joris Roos (Nov 16 2024 at 12:42):
(using Lean version 4.15.0-nightly-2024-11-15)
structure A where
p: Prop
q: True
structure B extends A where
q': p → True
example: B where
p := True ∧ True
q := by exact True.intro
q' := λ ⟨_,_⟩ ↦ True.intro
gives the unexpected kernel error (kernel) declaration has metavariables '_example'
Mysteriously (to me), any one of the following changes make the error disappear:
- replacing
by exact True.intro
byTrue.intro
- replacing
⟨_,_⟩
by_
- moving any of
p
,q
intoB
(orq'
intoA
)
Could someone shed some light on this?
Kim Morrison (Dec 03 2024 at 00:07):
Sorry about the slow reply on this. I wonder if this is the same issue as lean#5925.
Kim Morrison (Dec 03 2024 at 00:08):
If you want to open an issue, perhaps link to that one?
Joris Roos (Dec 10 2024 at 12:21):
Thanks, I opened a new issue: lean#6354
Kyle Miller (Dec 19 2024 at 00:50):
Last updated: May 02 2025 at 03:31 UTC