Skip to content

Commit

Permalink
upd doc
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist committed Jul 5, 2024
1 parent 95d7428 commit 08cc252
Showing 1 changed file with 6 additions and 10 deletions.
16 changes: 6 additions & 10 deletions theories/lebesgue_integral.v
Original file line number Diff line number Diff line change
Expand Up @@ -39,7 +39,8 @@ Require Import esum measure lebesgue_measure numfun realfun function_spaces.
(* *)
(* Detailed contents: *)
(* ```` *)
(* {mfun T >-> R} == type of real-valued measurable functions *)
(* {mfun aT >-> rT} == type of measurable functions *)
(* aT and rT are sigmaRingType's. *)
(* {sfun T >-> R} == type of simple functions *)
(* {nnsfun T >-> R} == type of non-negative simple functions *)
(* cst_nnsfun r == constant simple function *)
Expand Down Expand Up @@ -107,12 +108,8 @@ HB.mixin Record isMeasurableFun d d' (aT : sigmaRingType d) (rT : sigmaRingType
HB.structure Definition MeasurableFun d d' aT rT :=
{f of @isMeasurableFun d d' aT rT f}.

(* HB.mixin Record isMeasurableFun d (aT : measurableType d) (rT : realType) (f : aT -> rT) := { *)
(* measurable_funP : measurable_fun setT f *)
(* }. *)
(* #[global] Hint Resolve fimfun_inP : core. *)

(* HB.structure Definition MeasurableFun d aT rT := {f of @isMeasurableFun d aT rT f}. *)
Reserved Notation "{ 'mfun' aT >-> T }"
(at level 0, format "{ 'mfun' aT >-> T }").
Reserved Notation "[ 'mfun' 'of' f ]"
Expand Down Expand Up @@ -147,8 +144,6 @@ Notation "{ 'nnfun' aT >-> T }" := (@NonNegFun.type aT T) : form_scope.
Notation "[ 'nnfun' 'of' f ]" := [the {nnfun _ >-> _} of f] : form_scope.
#[global] Hint Extern 0 (is_true (0 <= _)) => solve [apply: fun_ge0] : core.

(* HB.structure Definition NonNegSimpleFun d (aT : measurableType d) (rT : realType) := *)

HB.structure Definition NonNegSimpleFun
d (aT : sigmaRingType d) (rT : realType) :=
{f of @SimpleFun d _ _ f & @NonNegFun aT rT f}.
Expand Down Expand Up @@ -291,10 +286,11 @@ End mfun.
Section mfun_realType.
Context {d} {aT : sigmaRingType d} {rT : realType}.

Let cst_mfun_subproof x : @isMeasurableFun d _ aT rT (cst x).
Proof. by split. Qed.
Let cst_mfun_subproof x : @measurable_fun d _ aT rT [set: aT] (cst x).
Proof. by []. Qed.

HB.instance Definition _ x := @cst_mfun_subproof x.
HB.instance Definition _ x := isMeasurableFun.Build d _ aT rT (cst x)
(@cst_mfun_subproof x).

HB.instance Definition _ := @isMeasurableFun.Build _ _ _ rT
(@normr rT rT) (@measurable_normr rT setT).
Expand Down

0 comments on commit 08cc252

Please sign in to comment.