Prerequisites
Description
The code below produces a PANIC at the first @[simp] and an internal exception #3 at the second one.
Context
set_option autoImplicit false
structure Foo where
foo := 37
variable {G : Foo}
def Foo.bar {U : Type} (f : Nat → Nat) := G.foo = G.foo
variable (C : G.bar baz)
include C
@[simp]
theorem quux : G.foo ↔ G.foo :=
sorry
@[simp]
theorem eggs : true :=
sorry
Steps to Reproduce
- Move the cursor to either simp
Expected behavior:: Probably some unknown identifier error depending on where the "real" error is occuring, but alternatively some error about metavariables without a backtrace if that's appropriate.
Actual behavior: : Observe a backtrace at the first one, and an internal exception at the second
Versions
[Output of #version or #eval Lean.versionString] 4.27.0-rc1
[OS version, if not using live.lean-lang.org.] macOS
Additional Information
Impact
Add 👍 to issues you consider important. If others are impacted by this issue, please ask them to add 👍 to it.