Skip to content

Commit

Permalink
adapt to hierarchy with subprob
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist committed Feb 12, 2023
1 parent 9038840 commit 8756b29
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 11 deletions.
10 changes: 1 addition & 9 deletions theories/kernel.v
Original file line number Diff line number Diff line change
Expand Up @@ -582,14 +582,6 @@ Arguments measurable_fun_xsection_integral {_ _ _ _ _} k l.
Arguments measurable_fun_integral_finite_kernel {_ _ _ _ _} k l.
Arguments measurable_fun_integral_sfinite_kernel {_ _ _ _ _} k l.

Section pdirac.
Context d (T : measurableType d) (R : realType).

HB.instance Definition _ x :=
isProbability.Build _ _ _ (@dirac _ T x R) (diracT R x).

End pdirac.

Section kdirac.
Context d d' (X : measurableType d) (Y : measurableType d') (R : realType).
Variable f : X -> Y.
Expand Down Expand Up @@ -825,7 +817,7 @@ by rewrite -{1}(@fineK _ (f x setT))// -EFinM divrr// ?unitfE fine_eq0.
Qed.

HB.instance Definition _ x :=
isProbability.Build _ _ _ (mnormalize x) (mnormalize1 x).
Measure_isProbability.Build _ _ _ (mnormalize x) (mnormalize1 x).

End mnormalize.

Expand Down
2 changes: 1 addition & 1 deletion theories/prob_lang.v
Original file line number Diff line number Diff line change
Expand Up @@ -71,7 +71,7 @@ rewrite /bernoulli/= /measure_add/= /msum 2!big_ord_recr/= big_ord0 add0e/=.
by rewrite /mscale/= !diracT !mule1 -EFinD onem1'.
Qed.

HB.instance Definition _ := @isProbability.Build _ _ R bernoulli bernoulli_setT.
HB.instance Definition _ := @Measure_isProbability.Build _ _ R bernoulli bernoulli_setT.

End bernoulli.

Expand Down
2 changes: 1 addition & 1 deletion theories/wip.v
Original file line number Diff line number Diff line change
Expand Up @@ -97,7 +97,7 @@ HB.instance Definition _ := isMeasure.Build _ _ _
Let mgauss01_setT : mgauss01 [set: _] = 1%E.
Proof. by rewrite /mgauss01 integral_gauss01_density. Qed.

HB.instance Definition _ := @isProbability.Build _ _ R mgauss01 mgauss01_setT.
HB.instance Definition _ := @Measure_isProbability.Build _ _ R mgauss01 mgauss01_setT.

Definition gauss01 := [the probability _ _ of mgauss01].

Expand Down

0 comments on commit 8756b29

Please sign in to comment.