diff options
author | Son HO | 2023-08-09 10:18:38 +0200 |
---|---|---|
committer | GitHub | 2023-08-09 10:18:38 +0200 |
commit | da97fc1e68d147439436ff883ac865a9cdeca18e (patch) | |
tree | 7d1165bcdd511f83555c63b29e6a24b8863bc1bf /tests/lean/Constants.lean | |
parent | 3d377976afe382a32f6ce718b473db5f016b1e47 (diff) | |
parent | fe8c303fef16d03ee17cd6af018296c0268e888c (diff) |
Merge pull request #34 from AeneasVerif/son_update_rustc
Update rustc to nightly-2023-06-02
Diffstat (limited to '')
-rw-r--r-- | tests/lean/Constants.lean | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/tests/lean/Constants.lean b/tests/lean/Constants.lean index ec07d0fe..51b415d6 100644 --- a/tests/lean/Constants.lean +++ b/tests/lean/Constants.lean @@ -9,7 +9,7 @@ namespace constants def x0_body : Result U32 := Result.ret (U32.ofInt 0) def x0_c : U32 := eval_global x0_body (by simp) -/- [core::num::u32::{9}::MAX] -/ +/- [core::num::u32::{8}::MAX] -/ def core_num_u32_max_body : Result U32 := Result.ret (U32.ofInt 4294967295) def core_num_u32_max_c : U32 := eval_global core_num_u32_max_body (by simp) |