Skip to content

Commit

Permalink
chore: update lean
Browse files Browse the repository at this point in the history
  • Loading branch information
digama0 committed Jul 31, 2023
1 parent 52223db commit 03139ed
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 3 deletions.
3 changes: 2 additions & 1 deletion Mathport/Syntax/Translate/Tactic/Mathlib/Padics.lean
Original file line number Diff line number Diff line change
Expand Up @@ -29,7 +29,8 @@ open Parser
`(tactic| init_ring $[using $(← liftM $ (← parse (tk "using" *> pExpr)?).mapM trExpr)]?)

@[tr_tactic ghost_simp] def trGhostSimp : TacM Syntax.Tactic := do
`(tactic| ghost_simp $[[$((← trSimpArgs (← parse simpArgList)).asNonempty),*]]?)
let args := (← trSimpArgs (← parse simpArgList)).asNonempty
`(tactic| ghost_simp $[[$args,*]]?)

@[tr_tactic witt_truncate_fun_tac] def trWittTruncateFunTac : TacM Syntax.Tactic :=
`(tactic| witt_truncate_fun_tac)
Expand Down
2 changes: 1 addition & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,7 @@
{"git":
{"url": "https://github.com/leanprover-community/mathlib4",
"subDir?": null,
"rev": "f39466cb99f0b941b72e1d918d139ef25a419023",
"rev": "dc89373908a65cd4807c248c566cbb75c18328f9",
"name": "mathlib",
"inputRev?": "master"}},
{"git":
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:nightly-2023-07-24
leanprover/lean4:nightly-2023-07-30

0 comments on commit 03139ed

Please sign in to comment.