Skip to content

Commit

Permalink
Adapt w.r.t. coq/coq#18909. (#108)
Browse files Browse the repository at this point in the history
  • Loading branch information
ppedrot authored Apr 9, 2024
1 parent ab93950 commit 9aaab98
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Common/Frame.v
Original file line number Diff line number Diff line change
Expand Up @@ -369,7 +369,7 @@ Module PO.
-> morph leB eqB leC eqC g -> morph leA eqA leC eqC (fun x => g (f x)).
Proof.
intros. destruct H, H0. constructor; intros.
- apply (PreO.morph_compose (leB := leB)); eauto using PreO. apply PreO.
- apply (PreO.morph_compose (leB := leB)); pose @PreO; eauto.
- solve_proper.
Qed.

Expand Down Expand Up @@ -453,7 +453,7 @@ Module PO.
- unfold pointwise_op. split; simpl in *; intros.
rewrite <- H0. rewrite <- H. apply H1.
rewrite H0. rewrite H. apply H1.
- unfold pointwise_op. eauto using le_antisym.
- unfold pointwise_op. intros; eapply le_antisym; eauto.
Qed.

Definition morph_pointwise {A B C} `{tC : t C leC eqC} (f : B -> A)
Expand Down

0 comments on commit 9aaab98

Please sign in to comment.