From aebbc43842ec0c49058b718c685e08edf11ce614 Mon Sep 17 00:00:00 2001 From: David Monniaux Date: Wed, 1 Apr 2020 16:15:54 +0200 Subject: route through LICMaux --- backend/LICM.v | 5 +---- 1 file changed, 1 insertion(+), 4 deletions(-) (limited to 'backend/LICM.v') diff --git a/backend/LICM.v b/backend/LICM.v index d45eef43..0a0a1c7d 100644 --- a/backend/LICM.v +++ b/backend/LICM.v @@ -3,10 +3,7 @@ Require Import AST Linking. Require Import Memory Registers Op RTL. Require Inject. -Definition gen_injections (f : function) (max_pc : node) (max_reg : reg): - PTree.t (list Inject.inj_instr) := PTree.empty (list Inject.inj_instr). - -Opaque gen_injections. +Axiom gen_injections : function -> node -> reg -> PTree.t (list Inject.inj_instr). Definition transf_program : program -> res program := Inject.transf_program gen_injections. -- cgit