Skip to content

Commit

Permalink
fixes for lean4#2973
Browse files Browse the repository at this point in the history
  • Loading branch information
kmill committed Nov 28, 2023
1 parent d3a1d25 commit ed2e76b
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions Qq/Match.lean
Original file line number Diff line number Diff line change
Expand Up @@ -248,8 +248,8 @@ partial def isIrrefutablePattern : Term → Bool

scoped elab "_comefrom" n:ident "do" b:doSeq " in " body:term : term <= expectedType => do
let _ ← extractBind expectedType
(← elabTerm (← `(?m)).1.stripPos none).mvarId!.assign expectedType
elabTerm (← `(have $n:ident : ?m := (do $b:doSeq); $body)) expectedType
let ty ← exprToSyntax expectedType
elabTerm (← `(have $n:ident : $ty := (do $b:doSeq); $body)) expectedType

scoped syntax "_comefrom" ident "do" doSeq : term
macro_rules | `(assert! (_comefrom $n do $b); $body) => `(_comefrom $n do $b in $body)
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.0.0
leanprover/lean4-pr-releases:pr-release-2973

0 comments on commit ed2e76b

Please sign in to comment.