-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathpsci_features.v
111 lines (107 loc) · 4.54 KB
/
psci_features.v
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
92
93
94
95
96
97
98
99
100
101
102
103
104
105
106
107
108
109
110
111
Require Import CodeDeps.
Require Import Ident.
Local Open Scope Z_scope.
Definition _psci_func_id := 1%positive.
Definition _rec := 2%positive.
Definition _rec__1 := 3%positive.
Definition _ret := 4%positive.
Definition _t'1 := 5%positive.
Definition _t'2 := 6%positive.
Definition _t'3 := 7%positive.
Definition _t'4 := 8%positive.
Definition _t'5 := 9%positive.
Definition _t'6 := 10%positive.
Definition _t'7 := 11%positive.
Definition _t'8 := 12%positive.
Definition _t'9 := 13%positive.
Definition psci_features_body :=
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Ssequence
(Sifthenelse (Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592513) tulong)
tint)
(Sset _t'1 (Econst_int (Int.repr 1) tint))
(Sset _t'1
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 3288334337) tulong)
tint) tbool)))
(Sifthenelse (Etempvar _t'1 tint)
(Sset _t'2 (Econst_int (Int.repr 1) tint))
(Sset _t'2
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592514) tulong)
tint) tbool))))
(Sifthenelse (Etempvar _t'2 tint)
(Sset _t'3 (Econst_int (Int.repr 1) tint))
(Sset _t'3
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592515) tulong) tint)
tbool))))
(Sifthenelse (Etempvar _t'3 tint)
(Sset _t'4 (Econst_int (Int.repr 1) tint))
(Sset _t'4
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 3288334339) tulong) tint)
tbool))))
(Sifthenelse (Etempvar _t'4 tint)
(Sset _t'5 (Econst_int (Int.repr 1) tint))
(Sset _t'5
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592516) tulong) tint)
tbool))))
(Sifthenelse (Etempvar _t'5 tint)
(Sset _t'6 (Econst_int (Int.repr 1) tint))
(Sset _t'6
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 3288334340) tulong) tint) tbool))))
(Sifthenelse (Etempvar _t'6 tint)
(Sset _t'7 (Econst_int (Int.repr 1) tint))
(Sset _t'7
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592520) tulong) tint) tbool))))
(Sifthenelse (Etempvar _t'7 tint)
(Sset _t'8 (Econst_int (Int.repr 1) tint))
(Sset _t'8
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592521) tulong) tint) tbool))))
(Sifthenelse (Etempvar _t'8 tint)
(Sset _t'9 (Econst_int (Int.repr 1) tint))
(Sset _t'9
(Ecast
(Ebinop Oeq (Etempvar _psci_func_id tuint)
(Econst_long (Int64.repr 2214592522) tulong) tint) tbool))))
(Sifthenelse (Etempvar _t'9 tint)
(Sset _ret (Econst_long (Int64.repr 0) tulong))
(Sset _ret (Econst_long (Int64.repr 4294967295) tulong))))
(Scall None
(Evar _set_psci_result_x0 (Tfunction (Tcons tulong Tnil) tvoid
cc_default)) ((Etempvar _ret tulong) :: nil)))
.
Definition f_psci_features := {|
fn_return := tvoid;
fn_callconv := cc_default;
fn_params := ((_rec, (tptr Tvoid)) ::
(_psci_func_id, tuint) :: nil);
fn_vars := nil;
fn_temps := ((_ret, tulong) :: (_t'9, tint) :: (_t'8, tint) ::
(_t'7, tint) :: (_t'6, tint) :: (_t'5, tint) ::
(_t'4, tint) :: (_t'3, tint) :: (_t'2, tint) ::
(_t'1, tint) :: nil);
fn_body := psci_features_body
|}.