Skip to content

Commit

Permalink
Fixed normal_rv_def
Browse files Browse the repository at this point in the history
  • Loading branch information
binghe committed Oct 3, 2024
1 parent e994112 commit f8c3ff1
Showing 1 changed file with 4 additions and 3 deletions.
7 changes: 4 additions & 3 deletions examples/probability/distributionScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -212,14 +212,15 @@ QED

Overload ext_normal_density = “\mu sig. Normal o normal_density mu sig o real”

Definition normal_measure :
Definition normal_measure_def :
normal_measure mu sig s =
pos_fn_integral ext_lborel (\x. ext_normal_density mu sig x * indicator_fn s x)
End

Definition normal_rv :
Definition normal_rv_def :
normal_rv X p mu sig <=> real_random_variable X p /\
distribution p X = normal_measure mu sig
!s. s IN subsets Borel ==>
distribution p X s = normal_measure mu sig s
End

val _ = export_theory ();
Expand Down

0 comments on commit f8c3ff1

Please sign in to comment.