Skip to content

Commit 084bf82

Browse files
committed
Work around COQBUG(rocq-prover/rocq#5481)
1 parent f6cfefc commit 084bf82

File tree

3 files changed

+5
-5
lines changed

3 files changed

+5
-5
lines changed

pcuic/theories/PCUICExpandLetsCorrectness.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1468,7 +1468,7 @@ Qed.
14681468
Lemma OnOne2All_map2_map_all {A B I I'} {P} {i : list I} {l l' : list A} (g : B -> I -> I') (f : A -> B) :
14691469
OnOne2All (fun i x y => P (g (f x) i) (f x) (f y)) i l l' -> OnOne2All P (map2 g (map f l) i) (map f l) (map f l').
14701470
Proof.
1471-
induction 1; simpl; constructor; try congruence. len.
1471+
induction 1; simpl; constructor; try congruence; try assumption. len.
14721472
now rewrite map2_length !map_length.
14731473
Qed.
14741474

@@ -5545,4 +5545,4 @@ Proof.
55455545
cbn in *.
55465546
now eapply expanded_expand_lets in etat.
55475547
Unshelve. all:eauto. destruct wfΣ; eauto.
5548-
Qed.
5548+
Qed.

pcuic/theories/PCUICParallelReduction.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -2220,7 +2220,7 @@ Section ParallelSubstitution.
22202220
rewrite !inst_inst_case_context_wf //.
22212221
eapply on_free_vars_ctx_inst_case_context; tea; solve_all.
22222222
eapply pred1_pred1_ctx in X7.
2223-
eapply on_contexts_app_inv => //. now rewrite /id.
2223+
eapply on_contexts_app_inv => //. now rewrite /id; (* congruence is enough in monomorphic mode, but we have to work around COQBUG(https://github.com/coq/coq/issues/5481) *) cbv [pcontext] in *; repeat destruct ?; cbn in *; subst; assumption.
22242224
eapply (on_contexts_length X).
22252225
rewrite /id. rewrite {2}H1.
22262226
apply: X6; tea. 3:now len.
@@ -2351,7 +2351,7 @@ Section ParallelSubstitution.
23512351
rewrite !inst_inst_case_context_wf //.
23522352
eapply on_free_vars_ctx_inst_case_context; tea; solve_all.
23532353
eapply pred1_pred1_ctx in X3 => //.
2354-
eapply on_contexts_app_inv => //. now rewrite /id.
2354+
eapply on_contexts_app_inv => //. now rewrite /id; (* congruence is enough in monomorphic mode, but we have to work around COQBUG(https://github.com/coq/coq/issues/5481) *) cbv [pcontext] in *; repeat destruct ?; cbn in *; subst; assumption.
23552355
eapply (on_contexts_length X). 2:len; lia.
23562356
now rewrite {2}H0.
23572357
+ solve_all. rewrite /inst_case_branch_context in a1 *.

template-pcuic/theories/PCUICToTemplateCorrectness.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1210,7 +1210,7 @@ Qed.
12101210
Lemma OnOne2All_map2_map_all {A B I I'} {P} {i : list I} {l l' : list A} (g : B -> I -> I') (f : A -> B) :
12111211
OnOne2All (fun i x y => P (g (f x) i) (f x) (f y)) i l l' -> OnOne2All P (map2 g (map f l) i) (map f l) (map f l').
12121212
Proof.
1213-
induction 1; simpl; constructor; try congruence. len.
1213+
induction 1; simpl; constructor; try congruence; try assumption. len.
12141214
now rewrite map2_length !map_length.
12151215
Qed.
12161216

0 commit comments

Comments
 (0)