From 6379f6291eea909426f074db67837b04a1dec9ae Mon Sep 17 00:00:00 2001 From: David Monniaux Date: Wed, 1 Apr 2020 14:24:05 +0200 Subject: attempt at compiling --- backend/LICMproof.v | 21 +++++++++++++++++++++ 1 file changed, 21 insertions(+) create mode 100644 backend/LICMproof.v (limited to 'backend/LICMproof.v') diff --git a/backend/LICMproof.v b/backend/LICMproof.v new file mode 100644 index 00000000..065a7f74 --- /dev/null +++ b/backend/LICMproof.v @@ -0,0 +1,21 @@ +Require Import Coqlib Maps Errors Integers Floats Lattice Kildall. +Require Import AST Linking. +Require Import Memory Registers Op RTL. +Require Import LICM. +Require Injectproof. + +Definition match_prog : program -> program -> Prop := + Injectproof.match_prog gen_injections. + +Section PRESERVATION. + + Variables prog tprog: program. + Hypothesis TRANSF: match_prog prog tprog. + + Theorem transf_program_correct : + Smallstep.forward_simulation (semantics prog) (semantics tprog). + Proof. + apply Injectproof.transf_program_correct with (gen_injections := gen_injections). + exact TRANSF. + Qed. +End PRESERVATION. -- cgit