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
{{ message }}
This repository has been archived by the owner on Oct 14, 2023. It is now read-only.
Reduced the issue to a self-contained, reproducible test case.
Description
[Description of the issue]
Steps to Reproduce
Create a Lean file with the following
section
parameter H : Type
def my_def := H
include H
lemma some_lemma
: Type :=
begin
clear H,
have := my_def,
exact this
end
end
lemma some_lemma'
: Type :=
begin
clear H,
have := _root_.my_def H,
exact this
end
Expected behavior: [What you expect to happen]
The two lemmas should fail for the same reason, "unknown identifier 'H'"
Actual behavior: [What actually happens]
In the first lemma, the script executes successfully and the resulting proof term is rejected with:
failed to add declaration to environment, it contains local constants
I believe to_expr should figure out that H is out of scope.
Reproduces how often: [What percentage of the time does it reproduce?]
100%
Prerequisites
or feature requests.
Description
[Description of the issue]
Steps to Reproduce
Create a Lean file with the following
Expected behavior: [What you expect to happen]
The two lemmas should fail for the same reason, "unknown identifier 'H'"
Actual behavior: [What actually happens]
In the first lemma, the script executes successfully and the resulting proof term is rejected with:
I believe
to_expr
should figure out thatH
is out of scope.Reproduces how often: [What percentage of the time does it reproduce?]
100%
Versions
I'm on OSX 10.13.2
Lean (version 3.3.1, commit 368f17d, RELEASE)
Additional Information
The text was updated successfully, but these errors were encountered: