From ee558407e59c6794daad70aab2e1e7794535367e Mon Sep 17 00:00:00 2001 From: Léo Gourdin Date: Mon, 17 May 2021 19:12:46 +0200 Subject: finishing RTLtoBTL --- scheduling/BTL.v | 18 ------------------ 1 file changed, 18 deletions(-) (limited to 'scheduling/BTL.v') diff --git a/scheduling/BTL.v b/scheduling/BTL.v index d55a0415..10a000a8 100644 --- a/scheduling/BTL.v +++ b/scheduling/BTL.v @@ -833,21 +833,3 @@ Lemma expand_correct ib: forall k, Proof. induction ib; simpl; intros; try autodestruct; auto. Qed. - -Lemma expand_None_correct ib: - is_expand (expand ib None). -Proof. - apply expand_correct; simpl; auto. -Qed. - -Definition expand_code (cfg: code): code := - (PTree.map (fun _ ib => {| entry:=expand ib.(entry) None; input_regs := ib.(input_regs) |}) cfg). - -Lemma expand_code_correct cfg pc ib : - (expand_code cfg)!pc=Some ib -> is_expand (ib.(entry)). -Proof. - unfold expand_code. - rewrite PTree.gmap. - destruct (cfg!pc); simpl; intros; try_simplify_someHyps. - apply expand_None_correct; auto. -Qed. -- cgit