summaryrefslogtreecommitdiff
path: root/tests/lean/Bitwise.lean
diff options
context:
space:
mode:
authorNadrieril2024-05-23 14:41:00 +0200
committerGuillaume Boisseau2024-05-24 14:24:38 +0200
commit25973ee8ef28e2d5b8a9b9ec3de4d6ff340db18b (patch)
tree07cd854559218325e030ac8c267720b0c5322251 /tests/lean/Bitwise.lean
parent4ce3e9c7c11744abae52d7a3ae1a3962395784be (diff)
Tweak a path
Diffstat (limited to '')
-rw-r--r--tests/lean/Bitwise.lean10
1 files changed, 5 insertions, 5 deletions
diff --git a/tests/lean/Bitwise.lean b/tests/lean/Bitwise.lean
index c13129f1..4ed56a0a 100644
--- a/tests/lean/Bitwise.lean
+++ b/tests/lean/Bitwise.lean
@@ -6,31 +6,31 @@ open Primitives
namespace bitwise
/- [bitwise::shift_u32]:
- Source: 'src/bitwise.rs', lines 3:0-3:31 -/
+ Source: 'tests/src/bitwise.rs', lines 3:0-3:31 -/
def shift_u32 (a : U32) : Result U32 :=
do
let t ← a >>> 16#usize
t <<< 16#usize
/- [bitwise::shift_i32]:
- Source: 'src/bitwise.rs', lines 10:0-10:31 -/
+ Source: 'tests/src/bitwise.rs', lines 10:0-10:31 -/
def shift_i32 (a : I32) : Result I32 :=
do
let t ← a >>> 16#isize
t <<< 16#isize
/- [bitwise::xor_u32]:
- Source: 'src/bitwise.rs', lines 17:0-17:37 -/
+ Source: 'tests/src/bitwise.rs', lines 17:0-17:37 -/
def xor_u32 (a : U32) (b : U32) : Result U32 :=
Result.ok (a ^^^ b)
/- [bitwise::or_u32]:
- Source: 'src/bitwise.rs', lines 21:0-21:36 -/
+ Source: 'tests/src/bitwise.rs', lines 21:0-21:36 -/
def or_u32 (a : U32) (b : U32) : Result U32 :=
Result.ok (a ||| b)
/- [bitwise::and_u32]:
- Source: 'src/bitwise.rs', lines 25:0-25:37 -/
+ Source: 'tests/src/bitwise.rs', lines 25:0-25:37 -/
def and_u32 (a : U32) (b : U32) : Result U32 :=
Result.ok (a &&& b)