You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
This was found by Joseph Rotella. The equation compiler fails to create a helper definition because of a universe error, even though the definition itself is sensible.
-- fails to create a helper definitiondeffoldr_cps {α β γ : Sort*} (g : α → β → β) (z : β) : list α → (β → γ) → γ
| list.nil k := k z
| (list.cons x xs) k := foldr_cps xs (λz', k (g x z'))
-- succeedsdeffoldr_cps' {α β γ : Sort*} (g : α → β → β) (z : β) (l : list α) : (β → γ) → γ :=
@list.rec_on α (λ _, (β → γ) → γ) l
(λ k : β → γ, k z)
(λ x xs r k, r (λ z', k (g x z')))
Prerequisites
Put an X between the brackets on this line if you have done all of the following:
Fixes half of the issue in #655, now it works if you specify the universe parameters explicitly.
If you don't specify them explicitly, then the auxiliary meta definition is declared before we have replaced the universe metavariables by u_1,u_2,... (called finalization), which happens at the very end of elaboration. Making that work as well would probably require large changes in the elaborator.
This was found by Joseph Rotella. The equation compiler fails to create a helper definition because of a universe error, even though the definition itself is sensible.
Prerequisites
or feature requests.
Description
[Description of the issue]
Steps to Reproduce
Expected behavior: [What you expect to happen]
Actual behavior: [What actually happens]
Reproduces how often: [What percentage of the time does it reproduce?]
Versions
You can get this information from copy and pasting the output of
lean --version
,please include the OS and what version of the OS you're running.
Additional Information
Any additional information, configuration or data that might be necessary to reproduce the issue.
The text was updated successfully, but these errors were encountered: