Skip to content

Commit

Permalink
Bump to leanprover/lean4:v4.5.0
Browse files Browse the repository at this point in the history
  • Loading branch information
shigoel committed Feb 1, 2024
1 parent 3a761c8 commit 88b16da
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Arm/Insts/Common.lean
Original file line number Diff line number Diff line change
Expand Up @@ -145,7 +145,7 @@ theorem M_divisible_by_esize_of_valid_bit_masks (immN : BitVec 1) (imms : BitVec
. simp
done

-- Resouces on Arm bitmask immediate:
-- Resources on Arm bitmask immediate:
-- https://developer.arm.com/documentation/dui0802/b/A64-General-Instructions/MOV--bitmask-immediate-
-- https://kddnewton.com/2022/08/11/aarch64-bitmask-immediates.html
-- Arm Implementation:
Expand Down
4 changes: 2 additions & 2 deletions Proofs/SHA512_AssocRepr.lean
Original file line number Diff line number Diff line change
Expand Up @@ -565,8 +565,8 @@ theorem sha512_block_armv8_new_program (s : ArmState)
simp only
simp [exec_inst, *]

unfold run
simp [stepi, h_pc]


sorry

end SHA512_proof
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.5.0-rc1
leanprover/lean4:v4.5.0

0 comments on commit 88b16da

Please sign in to comment.