Skip to content

Commit

Permalink
slight refactor of read_write_bytes_different
Browse files Browse the repository at this point in the history
  • Loading branch information
alexkeizer committed Oct 11, 2024
1 parent dcf0bce commit a221670
Showing 1 changed file with 5 additions and 6 deletions.
11 changes: 5 additions & 6 deletions Arm/Memory/MemoryProofs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -61,13 +61,12 @@ theorem Memory.read_write_bytes_different
induction n generalizing mem addr1 addr2
case zero => simp only [write_bytes]
case succ n ih =>
rw [write_bytes, ih ?h_sep]
case h_sep =>
show mem_separate addr1 addr1 (addr2 + 1#64)
(addr2 + 1#64 + BitVec.ofNat 64 (n - 1)) = true
have h_sep : mem_separate addr1 addr1 (addr2 + 1#64)
(addr2 + 1#64 + BitVec.ofNat 64 (n - 1)) := by
sorry
rw [Memory.read_write_different]
sorry
have h_neq : addr1 ≠ addr2 :=
mem_separate_starting_addresses_neq h
rw [write_bytes, ih h_sep, Memory.read_write_different h_neq]

theorem read_mem_of_write_mem_bytes_different (hn1 : n <= 2^64)
(h : mem_separate addr1 addr1 addr2 (addr2 + (BitVec.ofNat 64 (n - 1)))) :
Expand Down

0 comments on commit a221670

Please sign in to comment.