aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Machregs.v
diff options
context:
space:
mode:
Diffstat (limited to 'powerpc/Machregs.v')
-rw-r--r--powerpc/Machregs.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/powerpc/Machregs.v b/powerpc/Machregs.v
index b9af652a..62a4a0a5 100644
--- a/powerpc/Machregs.v
+++ b/powerpc/Machregs.v
@@ -206,6 +206,7 @@ Definition two_address_op (op: operation) : bool :=
Definition builtin_get_spr := ident_of_string "__builtin_get_spr".
Definition builtin_set_spr := ident_of_string "__builtin_set_spr".
+Definition builtin_prefetch := ident_of_string "__builtin_prefetch".
Definition builtin_constraints (ef: external_function) :
list builtin_arg_constraint :=
@@ -213,6 +214,7 @@ Definition builtin_constraints (ef: external_function) :
| EF_builtin id sg =>
if ident_eq id builtin_get_spr then OK_const :: nil
else if ident_eq id builtin_set_spr then OK_const :: OK_default :: nil
+ else if ident_eq id builtin_prefetch then OK_addrany :: OK_const :: OK_const :: nil
else nil
| EF_vload _ => OK_addrany :: nil
| EF_vstore _ => OK_addrany :: OK_default :: nil