aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GibleSeqgenproof.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2023-08-10 12:09:03 +0100
committerYann Herklotz <git@yannherklotz.com>2023-08-10 12:09:03 +0100
commit86e64fd05cea7b1da996701cd3653db5f471f8d1 (patch)
tree5cee338b89c4b1b2906cbf8e62d8f8dffdff0abb /src/hls/GibleSeqgenproof.v
parent4d62c7f35533ebd36ae4a0bdef6cd64fcc0be375 (diff)
downloadvericert-86e64fd05cea7b1da996701cd3653db5f471f8d1.tar.gz
vericert-86e64fd05cea7b1da996701cd3653db5f471f8d1.zip
Finish final forward simulation correctness
Diffstat (limited to 'src/hls/GibleSeqgenproof.v')
-rw-r--r--src/hls/GibleSeqgenproof.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/src/hls/GibleSeqgenproof.v b/src/hls/GibleSeqgenproof.v
index 7451510..1d1d4b7 100644
--- a/src/hls/GibleSeqgenproof.v
+++ b/src/hls/GibleSeqgenproof.v
@@ -253,6 +253,12 @@ whole execution (in one big step) of the basic block.
Definition match_prog (p: RTL.program) (tp: GibleSeq.program) :=
Linking.match_program (fun cu f tf => transl_fundef f = Errors.OK tf) eq p tp.
+ Lemma transf_program_match:
+ forall p tp, transl_program p = OK tp -> match_prog p tp.
+ Proof.
+ intros. apply Linking.match_transform_partial_program; auto.
+ Qed.
+
Context (TRANSL : match_prog prog tprog).
Lemma symbols_preserved: