summaryrefslogtreecommitdiff
path: root/tests/lean/External/Funs.lean
blob: e36987e0112f525c0cfbe2a5ecf61d3a6b97094a (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
-- THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS
-- [external]: function definitions
import Base
import External.Types
import External.ExternalFuns
open Primitives

namespace External

/- [external::swap] -/
def swap_fwd
  (T : Type) (x : T) (y : T) (st : State) : Result (State × Unit) :=
  do
    let (st0, _)  opaque_defs.core_mem_swap_fwd T x y st
    let (st1, _)  opaque_defs.core_mem_swap_back0 T x y st st0
    let (st2, _)  opaque_defs.core_mem_swap_back1 T x y st st1
    Result.ret (st2, ())

/- [external::swap] -/
def swap_back
  (T : Type) (x : T) (y : T) (st : State) (st0 : State) :
  Result (State × (T × T))
  :=
  do
    let (st1, _)  opaque_defs.core_mem_swap_fwd T x y st
    let (st2, x0)  opaque_defs.core_mem_swap_back0 T x y st st1
    let (_, y0)  opaque_defs.core_mem_swap_back1 T x y st st2
    Result.ret (st0, (x0, y0))

/- [external::test_new_non_zero_u32] -/
def test_new_non_zero_u32_fwd
  (x : U32) (st : State) : Result (State × core_num_nonzero_non_zero_u32_t) :=
  do
    let (st0, opt)  opaque_defs.core_num_nonzero_non_zero_u32_new_fwd x st
    opaque_defs.core_option_option_unwrap_fwd core_num_nonzero_non_zero_u32_t
      opt st0

/- [external::test_vec] -/
def test_vec_fwd : Result Unit :=
  do
    let v := vec_new U32
    let _  vec_push_back U32 v (U32.ofInt 0 (by intlit))
    Result.ret ()

/- Unit test for [external::test_vec] -/
#assert (test_vec_fwd == .ret ())

/- [external::custom_swap] -/
def custom_swap_fwd
  (T : Type) (x : T) (y : T) (st : State) : Result (State × T) :=
  do
    let (st0, _)  opaque_defs.core_mem_swap_fwd T x y st
    let (st1, x0)  opaque_defs.core_mem_swap_back0 T x y st st0
    let (st2, _)  opaque_defs.core_mem_swap_back1 T x y st st1
    Result.ret (st2, x0)

/- [external::custom_swap] -/
def custom_swap_back
  (T : Type) (x : T) (y : T) (st : State) (ret0 : T) (st0 : State) :
  Result (State × (T × T))
  :=
  do
    let (st1, _)  opaque_defs.core_mem_swap_fwd T x y st
    let (st2, _)  opaque_defs.core_mem_swap_back0 T x y st st1
    let (_, y0)  opaque_defs.core_mem_swap_back1 T x y st st2
    Result.ret (st0, (ret0, y0))

/- [external::test_custom_swap] -/
def test_custom_swap_fwd
  (x : U32) (y : U32) (st : State) : Result (State × Unit) :=
  do
    let (st0, _)  custom_swap_fwd U32 x y st
    Result.ret (st0, ())

/- [external::test_custom_swap] -/
def test_custom_swap_back
  (x : U32) (y : U32) (st : State) (st0 : State) :
  Result (State × (U32 × U32))
  :=
  custom_swap_back U32 x y st (U32.ofInt 1 (by intlit)) st0

/- [external::test_swap_non_zero] -/
def test_swap_non_zero_fwd (x : U32) (st : State) : Result (State × U32) :=
  do
    let (st0, _)  swap_fwd U32 x (U32.ofInt 0 (by intlit)) st
    let (st1, (x0, _))  swap_back U32 x (U32.ofInt 0 (by intlit)) st st0
    if x0 = (U32.ofInt 0 (by intlit))
    then Result.fail Error.panic
    else Result.ret (st1, x0)

end External