Skip to content

Commit

Permalink
revert change
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 22, 2023
1 parent 0831ae8 commit 1e11c50
Showing 1 changed file with 2 additions and 8 deletions.
10 changes: 2 additions & 8 deletions src/Lean/Meta/Tactic/Simp/Types.lean
Original file line number Diff line number Diff line change
Expand Up @@ -45,15 +45,9 @@ structure State where

abbrev SimpM := ReaderT Context $ StateRefT State MetaM

structure SavedState where
meta : Meta.SavedState
usedTheorems : UsedSimps

instance : MonadBacktrack SavedState SimpM where
saveState := return ⟨← Meta.saveState, (← get).usedTheorems⟩
restoreState s := do
s.meta.restore
modify fun t => { t with usedTheorems := s.usedTheorems }
saveState := Meta.saveState
restoreState s := s.restore

inductive Step where
| visit : Result → Step
Expand Down

0 comments on commit 1e11c50

Please sign in to comment.