From 4622f49fd089ae47d0c853343cb0a05f986c962a Mon Sep 17 00:00:00 2001 From: Xavier Leroy Date: Fri, 27 Mar 2015 08:55:05 +0100 Subject: Extend annotations so that they can keep track of global variables and local variables whose address is taken. - CminorSel, RTL: add "annot" instructions. - CminorSel to Asm: use type "annot_arg" for arguments of "annot" instructions. - AST, Events: simplify EF_annot because constants are now part of the arguments. Implementation is not complete yet. --- backend/Lineartyping.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'backend/Lineartyping.v') diff --git a/backend/Lineartyping.v b/backend/Lineartyping.v index ccf17e1e..c093b62d 100644 --- a/backend/Lineartyping.v +++ b/backend/Lineartyping.v @@ -76,7 +76,7 @@ Definition wt_instr (i: instruction) : bool := | Lbuiltin ef args res => subtype_list (proj_sig_res' (ef_sig ef)) (map mreg_type res) | Lannot ef args => - forallb loc_valid args + forallb loc_valid (params_of_annot_args args) | _ => true end. @@ -365,7 +365,7 @@ Qed. Lemma wt_state_annot: forall s f sp ef args c rs m, wt_state (State s f sp (Lannot ef args :: c) rs m) -> - forallb (loc_valid f) args = true. + forallb (loc_valid f) (params_of_annot_args args) = true. Proof. intros. inv H. simpl in WTC; InvBooleans. auto. Qed. -- cgit