-
Notifications
You must be signed in to change notification settings - Fork 726
Open
Labels
P-mediumWe may work on this issue if we find the timeWe may work on this issue if we find the timebugSomething isn't workingSomething isn't working
Description
Prerequisites
Please put an X between the brackets as you perform the following steps:
- Check that your issue is not already filed:
https://github.com/leanprover/lean4/issues - Reduce the issue to a minimal, self-contained, reproducible test case.
Avoid dependencies to Mathlib or Batteries. - Test your test case against the latest nightly release, for example on
https://live.lean-lang.org/#project=lean-nightly
(You can also use the settings there to switch to “Lean nightly”)
Description
The following lean code leads to a deep kernel reduction detected error in Lean.
theorem minimal6 : ∀ (x : BitVec 32),
((some x).bind fun x =>
(if False then none else some (x.sshiftRight 1)).bind fun x' =>
some (x'.sshiftRight 1))
= (some x) := by
intro x
simp only [Option.some_bind]
sorrySteps to Reproduce
- Copy into lean
- Observe the red line under the theorem name
Expected behavior: [Clear and concise description of what you expect to happen]
- simp should apply the lemma
- the proof should be marked as
sorrywith an orange line under the theorem name - no kernel error
Versions
"4.12.0-nightly-2024-10-15"
Impact
Add 👍 to issues you consider important. If others are impacted by this issue, please ask them to add 👍 to it.
This issue was reduced by @lfrenot.
tobiasgrosser, shigoel and GZGavinZhao
Metadata
Metadata
Assignees
Labels
P-mediumWe may work on this issue if we find the timeWe may work on this issue if we find the timebugSomething isn't workingSomething isn't working