summaryrefslogtreecommitdiff
path: root/powerpc/Machregs.v
diff options
context:
space:
mode:
Diffstat (limited to 'powerpc/Machregs.v')
-rw-r--r--powerpc/Machregs.v8
1 files changed, 7 insertions, 1 deletions
diff --git a/powerpc/Machregs.v b/powerpc/Machregs.v
index ce66e6a..d057dce 100644
--- a/powerpc/Machregs.v
+++ b/powerpc/Machregs.v
@@ -143,6 +143,12 @@ Definition destroyed_by_builtin (ef: external_function): list mreg :=
| _ => nil
end.
+Definition destroyed_by_setstack (ty: typ): list mreg :=
+ match ty with
+ | Tsingle => F13 :: nil
+ | _ => nil
+ end.
+
Definition destroyed_at_function_entry: list mreg :=
nil.
@@ -158,7 +164,7 @@ Definition mregs_for_builtin (ef: external_function): list (option mreg) * list
Global Opaque
destroyed_by_op destroyed_by_load destroyed_by_store
destroyed_by_cond destroyed_by_jumptable destroyed_by_builtin
- destroyed_at_function_entry temp_for_parent_frame
+ destroyed_by_setstack destroyed_at_function_entry temp_for_parent_frame
mregs_for_operation mregs_for_builtin.
(** Two-address operations. Return [true] if the first argument and