Skip to content

Commit

Permalink
Fixes for compatibility with Coq master
Browse files Browse the repository at this point in the history
  • Loading branch information
mattam82 committed May 22, 2024
1 parent 8bb76fb commit 526bc84
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions erasure-plugin/theories/ErasureCorrectness.v
Original file line number Diff line number Diff line change
Expand Up @@ -1878,7 +1878,7 @@ Section PCUICErase.
now eapply EEtaExpandedFix.expanded_isEtaExp. }
specialize (H0 H1).
eapply (obseq_lambdabox (Σ', f') (Σ', v'')) in obseq.
epose proof (ETransformPresAppLam.transform_lam _ _ _ (t := lambdabox_pres_app) (Σ', v'') prev H0).
epose proof (ETransformPresAppLam.transform_lam _ _ _ (t0 := lambdabox_pres_app) (Σ', v'') prev H0).
rewrite -obseq. exact H2. cbn. red; tauto.
Qed.

Expand Down Expand Up @@ -1933,7 +1933,7 @@ Section PCUICErase.
now eapply EEtaExpandedFix.expanded_isEtaExp. }
specialize (H0 H1).
eapply (obseq_lambdabox (Σ', f') (Σ', v'')) in obseq.
epose proof (ETransformPresAppLam.transform_lam _ _ _ (t := lambdabox_pres_app) (Σ', v'') prev H0).
epose proof (ETransformPresAppLam.transform_lam _ _ _ (t0 := lambdabox_pres_app) (Σ', v'') prev H0).
rewrite -obseq. exact H2. cbn. red; tauto.
Qed.

Expand Down Expand Up @@ -2455,7 +2455,7 @@ Section pipeline_theorem.
unshelve eapply (PCUICExpandLetsCorrectness.trans_wcbveval (cf := extraction_checker_flags) (Σ := (Σ.1, Σ.2))).
{ now eapply PCUICExpandLetsCorrectness.trans_wf. }
{ clear -HΣ typing''. now eapply PCUICClosedTyp.subject_closed in typing''. }
cbn. 2:cbn. 3:cbn. exact X0.
cbn. 2:cbn. exact X0.
now eapply (PCUICExpandLetsCorrectness.trans_axiom_free Σ).
pose proof (PCUICExpandLetsCorrectness.expand_lets_sound typing'').
rewrite PCUICExpandLetsCorrectness.trans_mkApps in X1. eapply X1.
Expand Down

0 comments on commit 526bc84

Please sign in to comment.