Skip to content

Commit

Permalink
doc: replay
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Feb 7, 2025
1 parent 273ae63 commit 1bc8941
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions src/Lean/Elab/Tactic/Try.lean
Original file line number Diff line number Diff line change
Expand Up @@ -290,6 +290,8 @@ where
-- Suboptimal combination. See comment at `isOnlyAndNonOnly`
return ()
let tac ← if let some tac2 ← mergeAll? tacs2 then
-- TODO: when merging tactics, there is a possibility the compressed version will not work.
-- TODO: if this is a big issue in practice, we should "replay" the tactic here.
`(tactic| $tac1:tactic <;> $tac2:tactic)
else
let tacs2 ← tacs2.mapM fun tac2 => `(tactic| · $tac2:tactic)
Expand Down

0 comments on commit 1bc8941

Please sign in to comment.