aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend
diff options
context:
space:
mode:
authorGaƫtan Gilbert <gaetan.gilbert@skyskimmer.net>2021-10-03 18:16:47 +0200
committerGitHub <noreply@github.com>2021-10-03 18:16:47 +0200
commita2a2529d78b86ece65cfc03fa8670538b85bc991 (patch)
tree83ff6fa2383b2bb69bd1066bd539e24e8c50a8f9 /cfrontend
parent11aaba64355ac8d912aee9b426476bf09c46bef1 (diff)
downloadcompcert-kvx-a2a2529d78b86ece65cfc03fa8670538b85bc991.tar.gz
compcert-kvx-a2a2529d78b86ece65cfc03fa8670538b85bc991.zip
Adapt to coq/coq#13837 ("apply with" does not rename arguments) (#417)
The change is backward compatible with Coq 8.9 to 8.13 (at least).
Diffstat (limited to 'cfrontend')
-rw-r--r--cfrontend/Ctyping.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/cfrontend/Ctyping.v b/cfrontend/Ctyping.v
index c930a407..97ed1ed3 100644
--- a/cfrontend/Ctyping.v
+++ b/cfrontend/Ctyping.v
@@ -2120,12 +2120,12 @@ Lemma wt_find_label:
wt_stmt ge e f.(fn_return) s' /\ wt_stmt_cont e f k'.
Proof.
intros lbl e f s0 WTS0. pattern s0.
- apply (wt_stmt_ind2 ge e f.(fn_return)) with
- (P0 := fun ls => wt_lblstmts ge e f.(fn_return) ls ->
+ apply (wt_stmt_ind2 ge e f.(fn_return) _
+ (fun ls => wt_lblstmts ge e f.(fn_return) ls ->
forall k s' k',
find_label_ls lbl ls k = Some (s', k') ->
wt_stmt_cont e f k ->
- wt_stmt ge e f.(fn_return) s' /\ wt_stmt_cont e f k');
+ wt_stmt ge e f.(fn_return) s' /\ wt_stmt_cont e f k'));
simpl; intros; try discriminate.
+ destruct (find_label lbl s1 (Kseq s2 k)) as [[sx kx] | ] eqn:F.
inv H3. eauto with ty.