Skip to content

Commit

Permalink
Merge pull request #35 from proux01/coq813
Browse files Browse the repository at this point in the history
Compile with Coq 8.13
  • Loading branch information
proux01 authored Jan 19, 2021
2 parents 9162e1c + 867631a commit f552e62
Show file tree
Hide file tree
Showing 3 changed files with 9 additions and 7 deletions.
1 change: 1 addition & 0 deletions .github/workflows/docker-action.yml
Original file line number Diff line number Diff line change
Expand Up @@ -17,6 +17,7 @@ jobs:
strategy:
matrix:
image:
- 'mathcomp/mathcomp:1.12.0-coq-8.13'
- 'mathcomp/mathcomp:1.12.0-coq-8.12'
- 'mathcomp/mathcomp:1.12.0-coq-8.11'
- 'mathcomp/mathcomp:1.12.0-coq-8.10'
Expand Down
2 changes: 2 additions & 0 deletions meta.yml
Original file line number Diff line number Diff line change
Expand Up @@ -72,6 +72,8 @@ dependencies:
[MathComp](https://math-comp.github.io) 1.11.0 or later
tested_coq_opam_versions:
- version: '1.12.0-coq-8.13'
repo: 'mathcomp/mathcomp'
- version: '1.12.0-coq-8.12'
repo: 'mathcomp/mathcomp'
- version: '1.12.0-coq-8.11'
Expand Down
13 changes: 6 additions & 7 deletions refinements/multipoly.v
Original file line number Diff line number Diff line change
Expand Up @@ -1314,8 +1314,8 @@ have -> : \sum_(m <- msupp p) f m p@_m
by rewrite Hf GRing.add0r GRing.scale0r GRing.subr0. }
eapply refines_apply.
{ eapply refines_apply; [by apply refine_mpoly_add_eff|].
eapply refines_apply; [|by apply trivial_refines; symmetry].
eapply refines_apply; [eapply ref_f|apply ref_m]. }
apply: (@refines_apply _ _ eq).
exact: trivial_refines. }
apply IH.
rewrite /pmcm /cm -Hc.
apply (rem_mpoly_eff Hq Hq' Hp ref_m).
Expand Down Expand Up @@ -1564,7 +1564,8 @@ apply refine_mpoly_sum_eff.
change (_ * _) with ((fun lq => c%:MP_[n] * mmap1 (tnth lq) m) lq).
eapply refines_apply; [|by apply ref_lq].
change (fun _ => _) with ((fun c lq => c%:MP_[n] * mmap1 (tnth lq) m) c).
eapply refines_apply; [|by apply trivial_refines; symmetry].
apply: (@refines_apply _ _ eq); last first.
{ exact: trivial_refines. }
change (fun _ => _) with ((fun m (c : T) lq => c%:MP_[n] * mmap1 (tnth lq) m) m).
eapply refines_apply; [apply refine_comp_monomial_eff|apply ref_m]. }
apply ref_p.
Expand Down Expand Up @@ -2138,10 +2139,8 @@ move=> K; inversion K.
eapply refines_apply; [apply refine_M_hrel_singleton|by apply trivial_refines]. }
eapply refines_apply; [eapply refines_apply|].
{ by apply refine_M_hrel_mpoly_mul_eff. }
{ eapply refines_apply; [|by apply trivial_refines; symmetry].
eapply refines_apply; first by apply refine_M_hrel_mpoly_exp_eff.
apply trivial_refines.
done. }
{ apply: (@refines_apply _ _ eq).
exact: trivial_refines. }
by apply IH; rewrite refinesE.
Qed.

Expand Down

0 comments on commit f552e62

Please sign in to comment.