aboutsummaryrefslogtreecommitdiffstats
path: root/backend/LICMproof.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-01 14:24:05 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-01 14:24:05 +0200
commit6379f6291eea909426f074db67837b04a1dec9ae (patch)
tree1d8a189c2863d7a9be543984badcd119ba4b5b3c /backend/LICMproof.v
parentd0590cab5ee32df395c129ee3edfa2dc3aaa202d (diff)
downloadcompcert-kvx-6379f6291eea909426f074db67837b04a1dec9ae.tar.gz
compcert-kvx-6379f6291eea909426f074db67837b04a1dec9ae.zip
attempt at compiling
Diffstat (limited to 'backend/LICMproof.v')
-rw-r--r--backend/LICMproof.v21
1 files changed, 21 insertions, 0 deletions
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.