Skip to content

Commit

Permalink
chore: add a dummy `evalTactic try simp_mem
Browse files Browse the repository at this point in the history
  • Loading branch information
bollu committed Sep 25, 2024
1 parent e4bf48b commit e1239bd
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions Tactics/Sym.lean
Original file line number Diff line number Diff line change
Expand Up @@ -330,6 +330,8 @@ since that would be way too expensive.
-/
def simpMem (_c : SymContext) (mvar : MVarId) : TacticM MVarId := do
/-
This should actually allow us to not need the follow processing in `Proofs/Popcount32`:
simp only [←Memory.mem_eq_iff_read_mem_bytes_eq] at *
simp only [memory_rules] at *
intro n addr h_separate
Expand Down

0 comments on commit e1239bd

Please sign in to comment.