diff options
author | Son HO | 2024-02-03 00:23:30 +0100 |
---|---|---|
committer | GitHub | 2024-02-03 00:23:30 +0100 |
commit | eb8bddcbd120f666f74023de9a23c48e1a55833d (patch) | |
tree | 1d8290e4b947e431c3d8d3a9f8575f23c3afe5e1 /tests/lean/Traits.lean | |
parent | 0960ad16838a43da3746f47cf5b640bfbb783d84 (diff) | |
parent | 9cc912e2414870df85ffc4dd346ade5dba2b5c37 (diff) |
Merge pull request #68 from AeneasVerif/son/update_lean
Update Lean to v4.6.0-rc1
Diffstat (limited to '')
-rw-r--r-- | tests/lean/Traits.lean | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/tests/lean/Traits.lean b/tests/lean/Traits.lean index d32aba86..3ef4febc 100644 --- a/tests/lean/Traits.lean +++ b/tests/lean/Traits.lean @@ -249,7 +249,7 @@ def traits.ToTypetraitsBoolWrapperTInst (T : Type) (ToTypeBoolTInst : ToType Source: 'src/traits.rs', lines 164:4-164:21 -/ def with_const_ty_len2_body : Result Usize := Result.ret 32#usize def with_const_ty_len2_c : Usize := - eval_global with_const_ty_len2_body (by simp) + eval_global with_const_ty_len2_body (by decide) /- Trait declaration: [traits::WithConstTy] Source: 'src/traits.rs', lines 161:0-161:39 -/ @@ -264,7 +264,7 @@ structure WithConstTy (Self : Type) (LEN : Usize) where /- [traits::{bool#8}::LEN1] Source: 'src/traits.rs', lines 175:4-175:21 -/ def bool_len1_body : Result Usize := Result.ret 12#usize -def bool_len1_c : Usize := eval_global bool_len1_body (by simp) +def bool_len1_c : Usize := eval_global bool_len1_body (by decide) /- [traits::{bool#8}::f]: Source: 'src/traits.rs', lines 180:4-180:39 -/ |