From 2a5715729f6454a9e664fcce52f269ee8c13e9e1 Mon Sep 17 00:00:00 2001 From: Cyril SIX Date: Mon, 7 Oct 2019 14:57:24 +0200 Subject: Itailcall --- backend/Duplicateproof.v | 10 ++++++++-- 1 file changed, 8 insertions(+), 2 deletions(-) (limited to 'backend/Duplicateproof.v') diff --git a/backend/Duplicateproof.v b/backend/Duplicateproof.v index 37c583df..aa605bea 100644 --- a/backend/Duplicateproof.v +++ b/backend/Duplicateproof.v @@ -26,8 +26,8 @@ Inductive match_inst (is_copy: node -> option node): instruction -> instruction is_copy n' = (Some n) -> match_inst is_copy (Istore m a lr r n) (Istore m a lr r n') | match_inst_call: forall n n' s ri lr r, is_copy n' = (Some n) -> match_inst is_copy (Icall s ri lr r n) (Icall s ri lr r n') - | match_inst_tailcall: forall n n' s ri lr, - is_copy n' = (Some n) -> match_inst is_copy (Itailcall s ri lr) (Itailcall s ri lr) + | match_inst_tailcall: forall s ri lr, + match_inst is_copy (Itailcall s ri lr) (Itailcall s ri lr) | match_inst_builtin: forall n n' ef la br, is_copy n' = (Some n) -> match_inst is_copy (Ibuiltin ef la br n) (Ibuiltin ef la br n') | match_inst_cond: forall ifso ifso' ifnot ifnot' c lr, @@ -114,6 +114,12 @@ Proof. destruct (Pos.eq_dec _ _); try discriminate. eapply verify_is_copy_correct_one. destruct x. eassumption. subst. constructor. +(* Itailcall *) + - destruct i'; try (inversion H; fail). + destruct (signature_eq _ _); try discriminate. + destruct (product_eq _ _ _ _); try discriminate. + destruct (list_eq_dec _ _ _); try discriminate. subst. clear H. + constructor. (* Ibuiltin *) - destruct i'; try (inversion H; fail). monadInv H. destruct (external_function_eq _ _); try discriminate. -- cgit