Skip to content

Commit

Permalink
rebase wrt 0.6.6
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist committed Jan 9, 2024
1 parent 6232e46 commit 4a191b6
Show file tree
Hide file tree
Showing 8 changed files with 47 additions and 253 deletions.
4 changes: 0 additions & 4 deletions .github/workflows/docker-action.yml
Original file line number Diff line number Diff line change
Expand Up @@ -15,11 +15,7 @@ jobs:
strategy:
matrix:
image:
- 'mathcomp/mathcomp:1.15.0-coq-8.14'
- 'mathcomp/mathcomp:1.15.0-coq-8.15'
- 'mathcomp/mathcomp:1.15.0-coq-8.16'
- 'mathcomp/mathcomp:1.16.0-coq-8.14'
- 'mathcomp/mathcomp:1.17.0-coq-8.15'
- 'mathcomp/mathcomp:1.17.0-coq-8.16'
- 'mathcomp/mathcomp:1.17.0-coq-8.17'
fail-fast: false
Expand Down
201 changes: 0 additions & 201 deletions .github/workflows/nix-action-8.14.yml

This file was deleted.

2 changes: 1 addition & 1 deletion coq-mathcomp-classical.opam
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,7 @@ the Coq proof-assistant and using the Mathematical Components library."""
build: [make "-C" "classical" "-j%{jobs}%"]
install: [make "-C" "classical" "install"]
depends: [
"coq" { (>= "8.14" & < "8.19~") | (= "dev") }
"coq" { (>= "8.16" & < "8.19~") | (= "dev") }
"coq-mathcomp-ssreflect" { (>= "1.13.0" & < "1.19~") | (= "dev") }
"coq-mathcomp-fingroup"
"coq-mathcomp-algebra"
Expand Down
10 changes: 5 additions & 5 deletions theories/lang_syntax.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,8 @@
Require Import String.
From HB Require Import structures.
From mathcomp Require Import all_ssreflect ssralg ssrnum ssrint interval.
From mathcomp.classical Require Import mathcomp_extra boolp classical_sets.
From mathcomp.classical Require Import functions cardinality fsbigop.
From mathcomp Require Import mathcomp_extra boolp classical_sets.
From mathcomp Require Import functions cardinality fsbigop.
Require Import signed reals ereal topology normedtype sequences esum measure.
Require Import lebesgue_measure numfun lebesgue_integral kernel prob_lang.
Require Import lang_syntax_util.
Expand Down Expand Up @@ -89,7 +89,7 @@ Proof. done. Qed.
Let mswap_sigma_additive x : semi_sigma_additive (mswap x).
Proof. exact: measure_semi_sigma_additive. Qed.

HB.instance Definition _ x := isMeasure.Build _ R _
HB.instance Definition _ x := isMeasure.Build _ _ R
(mswap x) (mswap0 x) (mswap_ge0 x) (@mswap_sigma_additive x).

Definition mkswap : _ -> {measure set Z -> \bar R} :=
Expand Down Expand Up @@ -185,7 +185,7 @@ Let T0 z : (T' z) set0 = 0. Proof. by []. Qed.
Let T_ge0 z x : 0 <= (T' z) x. Proof. by []. Qed.
Let T_semi_sigma_additive z : semi_sigma_additive (T' z).
Proof. exact: measure_semi_sigma_additive. Qed.
HB.instance Definition _ z := @isMeasure.Build _ R X (T' z) (T0 z) (T_ge0 z)
HB.instance Definition _ z := @isMeasure.Build _ X R (T' z) (T0 z) (T_ge0 z)
(@T_semi_sigma_additive z).

Let sfinT z : sfinite_measure (T' z). Proof. exact: sfinite_kernel_measure. Qed.
Expand All @@ -197,7 +197,7 @@ Let U0 z : (U' z) set0 = 0. Proof. by []. Qed.
Let U_ge0 z x : 0 <= (U' z) x. Proof. by []. Qed.
Let U_semi_sigma_additive z : semi_sigma_additive (U' z).
Proof. exact: measure_semi_sigma_additive. Qed.
HB.instance Definition _ z := @isMeasure.Build _ R Y (U' z) (U0 z) (U_ge0 z)
HB.instance Definition _ z := @isMeasure.Build _ Y R (U' z) (U0 z) (U_ge0 z)
(@U_semi_sigma_additive z).

Let sfinU z : sfinite_measure (U' z). Proof. exact: sfinite_kernel_measure. Qed.
Expand Down
Loading

0 comments on commit 4a191b6

Please sign in to comment.