summaryrefslogtreecommitdiff
path: root/tests/lean/Paper.lean
diff options
context:
space:
mode:
authorNadrieril2024-05-24 15:48:27 +0200
committerNadrieril2024-05-24 16:11:59 +0200
commit37e8a0f5ff7d964eb9525fef765b38e44f79302b (patch)
tree1a45ea3fdd5f462cf57c5dcc07b988c62749c7cd /tests/lean/Paper.lean
parent4d3778bea3112168645efc03308056ec341abb5f (diff)
Update test outputs
Diffstat (limited to 'tests/lean/Paper.lean')
-rw-r--r--tests/lean/Paper.lean18
1 files changed, 9 insertions, 9 deletions
diff --git a/tests/lean/Paper.lean b/tests/lean/Paper.lean
index bede3dd9..e98ada42 100644
--- a/tests/lean/Paper.lean
+++ b/tests/lean/Paper.lean
@@ -6,12 +6,12 @@ open Primitives
namespace paper
/- [paper::ref_incr]:
- Source: 'tests/src/paper.rs', lines 4:0-4:28 -/
+ Source: 'tests/src/paper.rs', lines 6:0-6:28 -/
def ref_incr (x : I32) : Result I32 :=
x + 1#i32
/- [paper::test_incr]:
- Source: 'tests/src/paper.rs', lines 8:0-8:18 -/
+ Source: 'tests/src/paper.rs', lines 10:0-10:18 -/
def test_incr : Result Unit :=
do
let x ← ref_incr 0#i32
@@ -23,7 +23,7 @@ def test_incr : Result Unit :=
#assert (test_incr == Result.ok ())
/- [paper::choose]:
- Source: 'tests/src/paper.rs', lines 15:0-15:70 -/
+ Source: 'tests/src/paper.rs', lines 17:0-17:70 -/
def choose
(T : Type) (b : Bool) (x : T) (y : T) :
Result (T × (T → Result (T × T)))
@@ -35,7 +35,7 @@ def choose
Result.ok (y, back)
/- [paper::test_choose]:
- Source: 'tests/src/paper.rs', lines 23:0-23:20 -/
+ Source: 'tests/src/paper.rs', lines 25:0-25:20 -/
def test_choose : Result Unit :=
do
let (z, choose_back) ← choose I32 true 0#i32 0#i32
@@ -55,13 +55,13 @@ def test_choose : Result Unit :=
#assert (test_choose == Result.ok ())
/- [paper::List]
- Source: 'tests/src/paper.rs', lines 35:0-35:16 -/
+ Source: 'tests/src/paper.rs', lines 37:0-37:16 -/
inductive List (T : Type) :=
| Cons : T → List T → List T
| Nil : List T
/- [paper::list_nth_mut]:
- Source: 'tests/src/paper.rs', lines 42:0-42:67 -/
+ Source: 'tests/src/paper.rs', lines 44:0-44:67 -/
divergent def list_nth_mut
(T : Type) (l : List T) (i : U32) : Result (T × (T → Result (List T))) :=
match l with
@@ -83,7 +83,7 @@ divergent def list_nth_mut
| List.Nil => Result.fail .panic
/- [paper::sum]:
- Source: 'tests/src/paper.rs', lines 57:0-57:32 -/
+ Source: 'tests/src/paper.rs', lines 59:0-59:32 -/
divergent def sum (l : List I32) : Result I32 :=
match l with
| List.Cons x tl => do
@@ -92,7 +92,7 @@ divergent def sum (l : List I32) : Result I32 :=
| List.Nil => Result.ok 0#i32
/- [paper::test_nth]:
- Source: 'tests/src/paper.rs', lines 68:0-68:17 -/
+ Source: 'tests/src/paper.rs', lines 70:0-70:17 -/
def test_nth : Result Unit :=
do
let l := List.Cons 3#i32 List.Nil
@@ -109,7 +109,7 @@ def test_nth : Result Unit :=
#assert (test_nth == Result.ok ())
/- [paper::call_choose]:
- Source: 'tests/src/paper.rs', lines 76:0-76:44 -/
+ Source: 'tests/src/paper.rs', lines 78:0-78:44 -/
def call_choose (p : (U32 × U32)) : Result U32 :=
do
let (px, py) := p