Skip to content

Commit

Permalink
Merge pull request #1081 from mrhaandi/faster-PCUICSR
Browse files Browse the repository at this point in the history
faster PCUICSR
  • Loading branch information
mattam82 authored Jun 12, 2024
2 parents 7f820b6 + be63a88 commit b9739c1
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions pcuic/theories/PCUICSR.v
Original file line number Diff line number Diff line change
Expand Up @@ -1626,7 +1626,7 @@ Proof.

- (* LetIn value *)
assert (X1' : lift_typing typing Σ Γ (j_vdef na r b_ty)).
{ unshelve eapply lift_judgment_SR with (1 := X1); tea. firstorder. }
{ unshelve eapply lift_judgment_SR with (1 := X1); tea. now constructor; [|right]. }
eapply type_Cumul_alt.
econstructor; eauto.
unshelve eapply (closed_context_conversion _ typeb'). pcuic.
Expand All @@ -1639,7 +1639,7 @@ Proof.

- (* LetIn type annotation *)
assert (X1' : lift_typing typing Σ Γ (j_vdef na b r)).
{ unshelve eapply lift_judgment_SR with (1 := X1); tea. firstorder. }
{ unshelve eapply lift_judgment_SR with (1 := X1); tea. now constructor; [|left]. }
eapply type_Cumul_alt.
econstructor; eauto.
unshelve eapply (closed_context_conversion _ typeb'). pcuic.
Expand Down

0 comments on commit b9739c1

Please sign in to comment.