From 5ad466befa609df178f04886484ee38b1a9c44ed Mon Sep 17 00:00:00 2001 From: Xavier Leroy Date: Thu, 23 Apr 2015 14:49:30 +0200 Subject: Take asm clobbers into account for determining callee-save registers used. --- backend/Bounds.v | 7 ++++++- 1 file changed, 6 insertions(+), 1 deletion(-) (limited to 'backend/Bounds.v') diff --git a/backend/Bounds.v b/backend/Bounds.v index 249ff796..7528b66e 100644 --- a/backend/Bounds.v +++ b/backend/Bounds.v @@ -87,6 +87,8 @@ Section BOUNDS. Variable f: function. +Parameter mregs_of_clobber: list ident -> list mreg. + (** In the proof of the [Stacking] pass, we only need to bound the registers written by an instruction. Therefore, this function returns these registers, ignoring registers used only as @@ -101,6 +103,7 @@ Definition regs_of_instr (i: instruction) : list mreg := | Lstore chunk addr args src => nil | Lcall sig ros => nil | Ltailcall sig ros => nil + | Lbuiltin (EF_inline_asm txt typs clob) args res => res ++ mregs_of_clobber clob | Lbuiltin ef args res => res ++ destroyed_by_builtin ef | Lannot ef args => nil | Llabel lbl => nil @@ -351,7 +354,9 @@ Proof. (* call *) eapply size_arguments_bound; eauto. (* builtin *) - apply H1. apply in_or_app; auto. + apply H1. destruct e; apply in_or_app; auto. + change (destroyed_by_builtin (EF_inline_asm text sg clobbers)) with (@nil mreg) in H2. + simpl in H2; tauto. (* annot *) apply H0. rewrite slots_of_locs_charact; auto. Qed. -- cgit