Skip to content

Commit

Permalink
Make scripts more robust when using simp and solving the goal trivially.
Browse files Browse the repository at this point in the history
  • Loading branch information
mattam82 committed May 23, 2024
1 parent d1f8f55 commit d6e0f45
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 4 deletions.
2 changes: 1 addition & 1 deletion erasure/theories/EEtaExpanded.v
Original file line number Diff line number Diff line change
Expand Up @@ -719,7 +719,7 @@ Proof.
solve_all.
- eapply In_All in H. simp_eta.
move=> /andP[] etarel etav.
eapply EEtaExpanded.isEtaExp_mkApps_intro. simp_eta. solve_all.
eapply EEtaExpanded.isEtaExp_mkApps_intro. now simp_eta. solve_all.
- eapply In_All in H0. simp_eta.
move=> /andP[] etau etav.
eapply EEtaExpanded.isEtaExp_mkApps_intro; auto. solve_all.
Expand Down
2 changes: 1 addition & 1 deletion erasure/theories/Typed/OptimizeCorrectness.v
Original file line number Diff line number Diff line change
Expand Up @@ -3191,7 +3191,7 @@ Proof.
now eapply (isEtaExp_lift _ _ [_] []).
eapply IHm; eauto. now move/andP: etal.
eapply IHm. eapply (isEtaExp_mkApps_intro _ _ _ [_]).
now eapply (isEtaExp_lift _ _ [_] []). constructor; eauto. simp_eta.
now eapply (isEtaExp_lift _ _ [_] []). constructor; eauto. now simp_eta.
eapply IHm. eapply (isEtaExp_mkApps_intro _ _ _ [_]); eauto. constructor; eauto.
all:now move/andP: etal.
Qed.
Expand Down
5 changes: 3 additions & 2 deletions pcuic/theories/PCUICParallelReductionConfluence.v
Original file line number Diff line number Diff line change
Expand Up @@ -1785,7 +1785,7 @@ Section Rho.
erewrite H; trea.
+ simp rho. simpl. f_equal; eauto.
erewrite -> rho_rename_pred; tea => //.
simp rho.
now simp rho.
+ simp rho. simpl. simp rho. f_equal; eauto.
erewrite -> rho_rename_pred; tea => //.

Expand Down Expand Up @@ -1850,7 +1850,8 @@ Section Rho.
simp rho. simpl.
f_equal; auto.
erewrite rho_rename_pred; tea=> //.
now rewrite !map_map_compose in H0. simp rho.
now rewrite !map_map_compose in H0.
now simp rho.

- (* Proj construct/cofix reduction *)
simpl.
Expand Down

0 comments on commit d6e0f45

Please sign in to comment.