summaryrefslogtreecommitdiff
path: root/tests/lean/Bitwise.lean
diff options
context:
space:
mode:
Diffstat (limited to 'tests/lean/Bitwise.lean')
-rw-r--r--tests/lean/Bitwise.lean18
1 files changed, 9 insertions, 9 deletions
diff --git a/tests/lean/Bitwise.lean b/tests/lean/Bitwise.lean
index c8538aa2..7c47e3dd 100644
--- a/tests/lean/Bitwise.lean
+++ b/tests/lean/Bitwise.lean
@@ -5,31 +5,31 @@ open Primitives
namespace bitwise
-/- [bitwise::shift_u32]: forward function
+/- [bitwise::shift_u32]:
Source: 'src/bitwise.rs', lines 3:0-3:31 -/
def shift_u32 (a : U32) : Result U32 :=
do
- let t ← a >>> 16#usize
- t <<< 16#usize
+ let t ← a >>> 16#usize
+ t <<< 16#usize
-/- [bitwise::shift_i32]: forward function
+/- [bitwise::shift_i32]:
Source: 'src/bitwise.rs', lines 10:0-10:31 -/
def shift_i32 (a : I32) : Result I32 :=
do
- let t ← a >>> 16#isize
- t <<< 16#isize
+ let t ← a >>> 16#isize
+ t <<< 16#isize
-/- [bitwise::xor_u32]: forward function
+/- [bitwise::xor_u32]:
Source: 'src/bitwise.rs', lines 17:0-17:37 -/
def xor_u32 (a : U32) (b : U32) : Result U32 :=
Result.ret (a ^^^ b)
-/- [bitwise::or_u32]: forward function
+/- [bitwise::or_u32]:
Source: 'src/bitwise.rs', lines 21:0-21:36 -/
def or_u32 (a : U32) (b : U32) : Result U32 :=
Result.ret (a ||| b)
-/- [bitwise::and_u32]: forward function
+/- [bitwise::and_u32]:
Source: 'src/bitwise.rs', lines 25:0-25:37 -/
def and_u32 (a : U32) (b : U32) : Result U32 :=
Result.ret (a &&& b)