Skip to content

Commit 8a5e984

Browse files
committed
Work around COQBUG(rocq-prover/rocq#17168)
1 parent 084bf82 commit 8a5e984

File tree

1 file changed

+7
-7
lines changed

1 file changed

+7
-7
lines changed

safechecker/theories/PCUICEqualityDec.v

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -452,7 +452,7 @@ Proof.
452452
1: eapply (All2_All_mix_left H0), (All2_All_mix_right H3), All2_map_inv ;
453453
eassumption.
454454
now move=> x y [? []] /X.
455-
* destruct (reflect_eq_ctx (pcontext pr) (pcontext pr')) => //.
455+
* case: (reflect_eq_ctx (pcontext pr) (pcontext pr')) => //.
456456
* now destruct (r equ Re 0 X (preturn pr')) ; nodec ; subst.
457457
- move/andb_and => [/andb_and [/andb_and [ppars pinst] pctx] pret].
458458
intuition auto.
@@ -464,7 +464,7 @@ Proof.
464464
1: eapply (All2_All_mix_left H0), (All2_All_mix_right H3), All2_map_inv;
465465
eassumption.
466466
now move=> x y [? []] /X.
467-
* now destruct (reflect_eq_ctx (pcontext pr) (pcontext pr')).
467+
* move: pctx; case: (reflect_eq_ctx (pcontext pr) (pcontext pr')) => //.
468468
* now destruct (r _ _ 0 X (preturn pr')).
469469
Qed.
470470

@@ -639,7 +639,7 @@ Proof.
639639
2:{ rewrite andb_false_r /=.
640640
constructor. intros bot; inv bot; contradiction.
641641
}
642-
destruct Hr => /=.
642+
case: Hr => e' /=.
643643
2:{
644644
constructor. intro bot. inversion bot. subst.
645645
auto.
@@ -657,17 +657,17 @@ Proof.
657657
cbn - [eqb]. inversion X. subst.
658658
destruct a, b. cbn - [eqb eqb_binder_annots].
659659
destruct X0 as [onc onbod].
660-
destruct (reflect_eq_ctx bcontext bcontext0) => // /=.
660+
case: (reflect_eq_ctx bcontext bcontext0) => a // /=.
661661
2:{ constructor. intro bot. inversion bot. subst.
662-
inversion X3. subst. destruct X4. cbn in e1. subst.
662+
inversion X3. subst. destruct X4. cbn in *. subst.
663663
contradiction.
664664
}
665665
cbn - [eqb].
666666
pose proof (onbod equ Re 0 he bbody0) as hh. cbn in hh.
667-
destruct hh => //=.
667+
case: hh => //= [e1|f].
668668
2:{ constructor. intro bot. apply f. inversion bot. subst.
669669
inversion X3. subst. destruct X4. assumption. }
670-
cbn -[eqb eqb_binder_annots] in *. destruct (IHl X1 brs) => //.
670+
cbn -[eqb eqb_binder_annots] in *. case: (IHl X1 brs) => // [e2|f].
671671
2:{ constructor. intro bot. apply f. inversion bot. subst.
672672
inversion X3. subst. constructor; auto. }
673673
constructor. inversion e2. subst.

0 commit comments

Comments
 (0)