Skip to content

Commit

Permalink
Adapt to Coq PR #17993 fixing Coq bug #12521 about simpl failing on m…
Browse files Browse the repository at this point in the history
…utual fixpoints with parameters. (#94)
  • Loading branch information
herbelin authored Sep 3, 2023
1 parent 2bb593d commit ff204c0
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 2 deletions.
2 changes: 1 addition & 1 deletion src/Parsers/Reachable/ParenBalanced/MinimalOfCore.v
Original file line number Diff line number Diff line change
Expand Up @@ -305,7 +305,7 @@ Section cfg.
{ left.
eexists (PBNil _ _ _).
unfold pb'_productions__of__minimal_pb'_productions; simpl.
rewrite expand_size_of_pb'_productions.
try rewrite expand_size_of_pb'_productions. (* compensate Coq bug #12521 before its fix in #17993 *)
simpl_size_of.
omega. }
{ assert (size_of_pb'_production p0' < h') by exact (lt_helper_1 H_h).
Expand Down
2 changes: 1 addition & 1 deletion src/Parsers/Reachable/ParenBalancedHiding/MinimalOfCore.v
Original file line number Diff line number Diff line change
Expand Up @@ -342,7 +342,7 @@ Section cfg.
{ left.
eexists (PBHNil _ _ _ _).
unfold pbh'_productions__of__minimal_pbh'_productions; simpl.
rewrite expand_size_of_pbh'_productions.
try rewrite expand_size_of_pbh'_productions. (* compensate Coq bug #12521 before its fix in #17993 *)
simpl_size_of.
omega. }
{ assert (size_of_pbh'_production p0' < h') by exact (lt_helper_1 H_h).
Expand Down
1 change: 1 addition & 0 deletions src/Parsers/SimpleRecognizerCorrect.v
Original file line number Diff line number Diff line change
Expand Up @@ -177,6 +177,7 @@ Section convenience.
Proof.
pose proof (parse_nonterminal_correct (gcdata := simple_gencdata1) str nt).
pose proof (parse_nonterminal_correct (gcdata := simple_gencdata2) str nt).
Opaque simple_parse_of_item_correct.
t_parse_correct.
match goal with H : _ |- _ => rewrite to_of_nonterminal in H end.
{ assumption. }
Expand Down

0 comments on commit ff204c0

Please sign in to comment.