We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 4b44ee9 commit 6063d9dCopy full SHA for 6063d9d
src/Lean/Elab/Tactic/BVAckermannize.lean
@@ -53,8 +53,8 @@ with `?w` a literal `Nat`. -/
53
def ofExpr? (e : Expr) : MetaM (Option BVTy) := ofExpr?Aux e |>.run where
54
ofExpr?Aux (e : Expr) : OptionT MetaM BVTy :=
55
match_expr e.consumeMData with
56
- | bool => return bool
57
- | bitVec w => do
+ | Bool => return bool
+ | BitVec w => do
58
let w ← getNatValue? w
59
return bitVec w
60
| _ => OptionT.fail
0 commit comments