aboutsummaryrefslogtreecommitdiffstats
path: root/scheduling/RTLtoBTLproof.v
diff options
context:
space:
mode:
authorSylvain Boulmé <sylvain.boulme@univ-grenoble-alpes.fr>2021-05-08 07:31:05 +0200
committerSylvain Boulmé <sylvain.boulme@univ-grenoble-alpes.fr>2021-05-08 07:31:05 +0200
commita1cde0686dfb40595423f40ccc40e18de3539e52 (patch)
tree999f44305e17ff594d9896f81a98926a423ee747 /scheduling/RTLtoBTLproof.v
parent1d32156c5bc43f966abe2c12c317a27e092355c4 (diff)
downloadcompcert-kvx-a1cde0686dfb40595423f40ccc40e18de3539e52.tar.gz
compcert-kvx-a1cde0686dfb40595423f40ccc40e18de3539e52.zip
idee pour simplifier la preuve: restreindre le "right_assoc" en "expand" !
Diffstat (limited to 'scheduling/RTLtoBTLproof.v')
-rw-r--r--scheduling/RTLtoBTLproof.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/scheduling/RTLtoBTLproof.v b/scheduling/RTLtoBTLproof.v
index 7d58de5a..7c9fb456 100644
--- a/scheduling/RTLtoBTLproof.v
+++ b/scheduling/RTLtoBTLproof.v
@@ -6,6 +6,8 @@ Require Import Errors Linking RTLtoBTL.
Require Import Linking.
+(* TODO: remplacer "right_assoc" par "expand" ci-dessous *)
+
Record match_function dupmap (f:RTL.function) (tf: BTL.function): Prop := {
dupmap_correct: match_cfg dupmap (fn_code tf) (RTL.fn_code f);
dupmap_entrypoint: dupmap!(fn_entrypoint tf) = Some (RTL.fn_entrypoint f);