Skip to content

Commit

Permalink
Merge branch 'main' into cleanup-popcount
Browse files Browse the repository at this point in the history
  • Loading branch information
shigoel authored Sep 25, 2024
2 parents 2d5a84b + bbd3075 commit 8f7799d
Show file tree
Hide file tree
Showing 5 changed files with 797 additions and 178 deletions.
1 change: 1 addition & 0 deletions Arm/State.lean
Original file line number Diff line number Diff line change
Expand Up @@ -820,6 +820,7 @@ A variant of `write_mem` that directly talks about writes to memory, instead of
def Memory.write (addr : BitVec 64) (val : BitVec 8) (m : Memory) : Memory :=
write_store addr val m

@[state_simp_rules]
theorem ArmState.write_mem_eq_mem_write : (write_mem addr val s).mem = s.mem.write addr val := rfl

namespace Memory
Expand Down
177 changes: 0 additions & 177 deletions Proofs/Experiments/MemCpyVCG.lean

This file was deleted.

Loading

0 comments on commit 8f7799d

Please sign in to comment.