aboutsummaryrefslogtreecommitdiffstats
path: root/backend/LICM.v
blob: 787ce256294d21d81021bad1dc4ec228168d80a3 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
(* *************************************************************)
(*                                                             *)
(*             The Compcert verified compiler                  *)
(*                                                             *)
(*           David Monniaux     CNRS, VERIMAG                  *)
(*                                                             *)
(*  Copyright VERIMAG. All rights reserved.                    *)
(*  This file is distributed under the terms of the INRIA      *)
(*  Non-Commercial License Agreement.                          *)
(*                                                             *)
(* *************************************************************)

Require Import Coqlib Maps Errors Integers Floats Lattice Kildall.
Require Import AST Linking.
Require Import Memory Registers Op RTL.
Require Inject.

Axiom gen_injections : function -> node -> reg -> PTree.t (list Inject.inj_instr).

Definition transf_program : program -> res program :=
  Inject.transf_program gen_injections.