Skip to content

Commit

Permalink
chore: move to v4.9.0-rc1 (#44)
Browse files Browse the repository at this point in the history
* chore: adaptations for nightly-2024-05-09 (#43)

* move to v4.9.0-rc1
  • Loading branch information
kim-em authored Jun 7, 2024
1 parent 5315667 commit a7bfa63
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion Qq/Macro.lean
Original file line number Diff line number Diff line change
Expand Up @@ -495,7 +495,7 @@ def Impl.macro (t : Syntax) (expectedType : Expr) : TermElabM Expr := do
withProcessPostponed do withSynthesize do
let t ← Term.elabTerm t lastDecl.type
let t ← ensureHasType lastDecl.type t
synthesizeSyntheticMVars (mayPostpone := false)
synthesizeSyntheticMVars (postpone := .no)
if (← logUnassignedUsingErrorInfos (← getMVars t)) then
throwAbortTerm
lastId.assign t
Expand Down
2 changes: 1 addition & 1 deletion Qq/Match.lean
Original file line number Diff line number Diff line change
Expand Up @@ -172,7 +172,7 @@ def elabPat (pat : Term) (lctx : LocalContext) (localInsts : LocalInstances) (ty
let (pat, patVars) ← getPatVars pat #[]
let pat ← Lean.Elab.Term.elabTerm pat ty
let pat ← ensureHasType ty pat
synthesizeSyntheticMVars false
synthesizeSyntheticMVars (postpone := .no)
let pat ← instantiateMVars pat

let mctx ← getMCtx
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.6.0-rc1
leanprover/lean4:v4.9.0-rc1

0 comments on commit a7bfa63

Please sign in to comment.