Skip to content

Commit

Permalink
Beta-reduce, to not confuse delta?
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed Dec 11, 2024
1 parent f9b44aa commit 5382395
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Lean/Meta/ArgsPacker.lean
Original file line number Diff line number Diff line change
Expand Up @@ -198,7 +198,7 @@ return expression of type `(x : A) → (y : B) → … → (z : D) → R[(x,y,z)
-/
private partial def curry (varNames : Array Name) (e : Expr) : MetaM Expr := do
if varNames.isEmpty then
return .app e (mkConst ``Unit.unit)
return e.beta #[mkConst ``Unit.unit]
let type ← whnfForall (← inferType e)
unless type.isForall do
throwError "curryPSigma: expected forall type, got {type}"
Expand Down

0 comments on commit 5382395

Please sign in to comment.