aboutsummaryrefslogtreecommitdiffstats
path: root/scheduling/BTL.v
diff options
context:
space:
mode:
authorDavid Monniaux <David.Monniaux@univ-grenoble-alpes.fr>2021-12-01 13:18:32 +0100
committerDavid Monniaux <David.Monniaux@univ-grenoble-alpes.fr>2021-12-01 14:53:56 +0100
commita781244930ababd25e40c40e8df8bd437f3fbf8c (patch)
treeb5222bc32623c7ec58c66178f22afc3c9a2e065f /scheduling/BTL.v
parent20cdd9c6c3962f7bec5c85719cfa7b0ee22f0100 (diff)
parenta79f0f99831aa0b0742bf7cce459cc9353bd7cd0 (diff)
downloadcompcert-kvx-a781244930ababd25e40c40e8df8bd437f3fbf8c.tar.gz
compcert-kvx-a781244930ababd25e40c40e8df8bd437f3fbf8c.zip
Merge remote-tracking branch 'absint/master' into towards_3.10
Mostly changes in PTree
Diffstat (limited to 'scheduling/BTL.v')
-rw-r--r--scheduling/BTL.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/scheduling/BTL.v b/scheduling/BTL.v
index c10b8ac2..b3895768 100644
--- a/scheduling/BTL.v
+++ b/scheduling/BTL.v
@@ -419,8 +419,7 @@ Lemma transfer_regs_dead inputs rs r:
~List.In r inputs -> (transfer_regs inputs rs)#r = Vundef.
Proof.
unfold transfer_regs; induction inputs; simpl; intuition subst.
- - rewrite Regmap.gi; auto.
- - rewrite Regmap.gso; auto.
+ rewrite Regmap.gso; auto.
Qed.
Fixpoint union_inputs (f:function) (tbl: list exit): Regset.t :=