Skip to content

Commit

Permalink
complete the casino example
Browse files Browse the repository at this point in the history
- new version of Bernoulli
- cleaning
  • Loading branch information
affeldt-aist committed May 2, 2024
1 parent 1091c8f commit 5f48ff4
Show file tree
Hide file tree
Showing 12 changed files with 3,485 additions and 3,007 deletions.
2 changes: 1 addition & 1 deletion _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -57,7 +57,7 @@ theories/lang_syntax_util.v
theories/lang_syntax_toy.v
theories/lang_syntax.v
theories/lang_syntax_examples.v
theories/lang_syntax_examples_wip.v
theories/lang_syntax_table_game.v
theories/altreals/xfinmap.v
theories/altreals/discrete.v
theories/altreals/realseq.v
Expand Down
2 changes: 1 addition & 1 deletion theories/Make
Original file line number Diff line number Diff line change
Expand Up @@ -47,7 +47,7 @@ lang_syntax_util.v
lang_syntax_toy.v
lang_syntax.v
lang_syntax_examples.v
lang_syntax_examples_wip.v
lang_syntax_table_game.v
altreals/xfinmap.v
altreals/discrete.v
altreals/realseq.v
Expand Down
6 changes: 3 additions & 3 deletions theories/kernel.v
Original file line number Diff line number Diff line change
Expand Up @@ -506,7 +506,7 @@ Variable k : X * Y -> \bar R.

Lemma measurable_fun_xsection_integral
(l : X -> {measure set Y -> \bar R})
(k_ : ({nnsfun [the measurableType _ of X * Y] >-> R})^nat)
(k_ : {nnsfun (X * Y) >-> R}^nat)
(ndk_ : nondecreasing_seq (k_ : (X * Y -> R)^nat))
(k_k : forall z, (k_ n z)%:E @[n --> \oo] --> k z) :
(forall n r,
Expand Down Expand Up @@ -614,7 +614,7 @@ Qed.
HB.instance Definition _ := isKernel.Build _ _ _ _ _ (kdirac mf)
measurable_fun_kdirac.

Let kdirac_prob x : kdirac mf x setT = 1.
Let kdirac_prob x : kdirac mf x [set: Y] = 1.
Proof. by rewrite /kdirac/= diracT. Qed.

HB.instance Definition _ := Kernel_isProbability.Build _ _ _ _ _
Expand Down Expand Up @@ -722,7 +722,7 @@ Context d d' (X : measurableType d) (Y : measurableType d') (R : realType).
Variable f : R.-ker X ~> Y.

Definition knormalize (P : probability Y R) : X -> {measure set Y -> \bar R} :=
fun x => [the measure _ _ of mnormalize (f x) P].
fun x => mnormalize (f x) P.

Let measurable_knormalize (P : probability Y R) U :
measurable U -> measurable_fun [set: X] (knormalize P ^~ U).
Expand Down
Loading

0 comments on commit 5f48ff4

Please sign in to comment.