summaryrefslogtreecommitdiff
path: root/tests/lean/NoNestedBorrows.lean
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--tests/lean/NoNestedBorrows.lean152
1 files changed, 76 insertions, 76 deletions
diff --git a/tests/lean/NoNestedBorrows.lean b/tests/lean/NoNestedBorrows.lean
index aa782009..b8fbcff0 100644
--- a/tests/lean/NoNestedBorrows.lean
+++ b/tests/lean/NoNestedBorrows.lean
@@ -82,9 +82,9 @@ def test3 : Result Unit :=
let x ← get_max 4#u32 3#u32
let y ← get_max 10#u32 11#u32
let z ← x + y
- if ¬ (z = 15#u32)
- then Result.fail .panic
- else Result.ok ()
+ if z = 15#u32
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test3] -/
#assert (test3 == Result.ok ())
@@ -94,9 +94,9 @@ def test3 : Result Unit :=
def test_neg1 : Result Unit :=
do
let y ← -. 3#i32
- if ¬ (y = (-3)#i32)
- then Result.fail .panic
- else Result.ok ()
+ if y = (-3)#i32
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_neg1] -/
#assert (test_neg1 == Result.ok ())
@@ -104,9 +104,9 @@ def test_neg1 : Result Unit :=
/- [no_nested_borrows::refs_test1]:
Source: 'tests/src/no_nested_borrows.rs', lines 97:0-97:19 -/
def refs_test1 : Result Unit :=
- if ¬ (1#i32 = 1#i32)
- then Result.fail .panic
- else Result.ok ()
+ if 1#i32 = 1#i32
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::refs_test1] -/
#assert (refs_test1 == Result.ok ())
@@ -114,17 +114,17 @@ def refs_test1 : Result Unit :=
/- [no_nested_borrows::refs_test2]:
Source: 'tests/src/no_nested_borrows.rs', lines 108:0-108:19 -/
def refs_test2 : Result Unit :=
- if ¬ (2#i32 = 2#i32)
- then Result.fail .panic
- else
- if ¬ (0#i32 = 0#i32)
- then Result.fail .panic
- else
- if ¬ (2#i32 = 2#i32)
- then Result.fail .panic
- else if ¬ (2#i32 = 2#i32)
- then Result.fail .panic
- else Result.ok ()
+ if 2#i32 = 2#i32
+ then
+ if 0#i32 = 0#i32
+ then
+ if 2#i32 = 2#i32
+ then if 2#i32 = 2#i32
+ then Result.ok ()
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::refs_test2] -/
#assert (refs_test2 == Result.ok ())
@@ -144,9 +144,9 @@ def test_box1 : Result Unit :=
let (_, deref_mut_back) ← alloc.boxed.Box.deref_mut I32 0#i32
let b ← deref_mut_back 1#i32
let x ← alloc.boxed.Box.deref I32 b
- if ¬ (x = 1#i32)
- then Result.fail .panic
- else Result.ok ()
+ if x = 1#i32
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_box1] -/
#assert (test_box1 == Result.ok ())
@@ -175,9 +175,9 @@ def test_panic (b : Bool) : Result Unit :=
def test_copy_int : Result Unit :=
do
let y ← copy_int 0#i32
- if ¬ (0#i32 = y)
- then Result.fail .panic
- else Result.ok ()
+ if 0#i32 = y
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_copy_int] -/
#assert (test_copy_int == Result.ok ())
@@ -194,9 +194,9 @@ def is_cons (T : Type) (l : List T) : Result Bool :=
def test_is_cons : Result Unit :=
do
let b ← is_cons I32 (List.Cons 0#i32 List.Nil)
- if ¬ b
- then Result.fail .panic
- else Result.ok ()
+ if b
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_is_cons] -/
#assert (test_is_cons == Result.ok ())
@@ -214,9 +214,9 @@ def test_split_list : Result Unit :=
do
let p ← split_list I32 (List.Cons 0#i32 List.Nil)
let (hd, _) := p
- if ¬ (hd = 0#i32)
- then Result.fail .panic
- else Result.ok ()
+ if hd = 0#i32
+ then Result.ok ()
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_split_list] -/
#assert (test_split_list == Result.ok ())
@@ -239,16 +239,16 @@ def choose_test : Result Unit :=
do
let (z, choose_back) ← choose I32 true 0#i32 0#i32
let z1 ← z + 1#i32
- if ¬ (z1 = 1#i32)
- then Result.fail .panic
- else
+ if z1 = 1#i32
+ then
do
let (x, y) ← choose_back z1
- if ¬ (x = 1#i32)
- then Result.fail .panic
- else if ¬ (y = 0#i32)
- then Result.fail .panic
- else Result.ok ()
+ if x = 1#i32
+ then if y = 0#i32
+ then Result.ok ()
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::choose_test] -/
#assert (choose_test == Result.ok ())
@@ -343,42 +343,42 @@ def test_list_functions : Result Unit :=
let l := List.Cons 2#i32 List.Nil
let l1 := List.Cons 1#i32 l
let i ← list_length I32 (List.Cons 0#i32 l1)
- if ¬ (i = 3#u32)
- then Result.fail .panic
- else
+ if i = 3#u32
+ then
do
let i1 ← list_nth_shared I32 (List.Cons 0#i32 l1) 0#u32
- if ¬ (i1 = 0#i32)
- then Result.fail .panic
- else
+ if i1 = 0#i32
+ then
do
let i2 ← list_nth_shared I32 (List.Cons 0#i32 l1) 1#u32
- if ¬ (i2 = 1#i32)
- then Result.fail .panic
- else
+ if i2 = 1#i32
+ then
do
let i3 ← list_nth_shared I32 (List.Cons 0#i32 l1) 2#u32
- if ¬ (i3 = 2#i32)
- then Result.fail .panic
- else
+ if i3 = 2#i32
+ then
do
let (_, list_nth_mut_back) ←
list_nth_mut I32 (List.Cons 0#i32 l1) 1#u32
let ls ← list_nth_mut_back 3#i32
let i4 ← list_nth_shared I32 ls 0#u32
- if ¬ (i4 = 0#i32)
- then Result.fail .panic
- else
+ if i4 = 0#i32
+ then
do
let i5 ← list_nth_shared I32 ls 1#u32
- if ¬ (i5 = 3#i32)
- then Result.fail .panic
- else
+ if i5 = 3#i32
+ then
do
let i6 ← list_nth_shared I32 ls 2#u32
- if ¬ (i6 = 2#i32)
- then Result.fail .panic
- else Result.ok ()
+ if i6 = 2#i32
+ then Result.ok ()
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_list_functions] -/
#assert (test_list_functions == Result.ok ())
@@ -453,26 +453,26 @@ def test_constants : Result Unit :=
do
let swt ← new_tuple1
let (i, _) := swt.p
- if ¬ (i = 1#u32)
- then Result.fail .panic
- else
+ if i = 1#u32
+ then
do
let swt1 ← new_tuple2
let (i1, _) := swt1.p
- if ¬ (i1 = 1#i16)
- then Result.fail .panic
- else
+ if i1 = 1#i16
+ then
do
let swt2 ← new_tuple3
let (i2, _) := swt2.p
- if ¬ (i2 = 1#u64)
- then Result.fail .panic
- else
+ if i2 = 1#u64
+ then
do
let swp ← new_pair1
- if ¬ (swp.p.x = 1#u32)
- then Result.fail .panic
- else Result.ok ()
+ if swp.p.x = 1#u32
+ then Result.ok ()
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
+ else Result.fail .panic
/- Unit test for [no_nested_borrows::test_constants] -/
#assert (test_constants == Result.ok ())
@@ -489,9 +489,9 @@ def test_weird_borrows1 : Result Unit :=
Source: 'tests/src/no_nested_borrows.rs', lines 407:0-407:37 -/
def test_mem_replace (px : U32) : Result U32 :=
let (y, _) := core.mem.replace U32 px 1#u32
- if ¬ (y = 0#u32)
- then Result.fail .panic
- else Result.ok 2#u32
+ if y = 0#u32
+ then Result.ok 2#u32
+ else Result.fail .panic
/- [no_nested_borrows::test_shared_borrow_bool1]:
Source: 'tests/src/no_nested_borrows.rs', lines 414:0-414:47 -/