Skip to content

Commit f132015

Browse files
committed
fixing hoelder.v after rebase
1 parent 86dccb4 commit f132015

File tree

2 files changed

+2
-20
lines changed

2 files changed

+2
-20
lines changed

theories/hoelder.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -43,7 +43,7 @@ HB.lock Definition Lnorm {d} {T : measurableType d} {R : realType}
4343
mu (f @^-1` (setT `\ 0%R))
4444
else
4545
(\int[mu]_x (`|f x| `^ p)%:E) `^ p^-1)%E
46-
| +oo%E => (if mu [set: T] > 0 then ess_sup mu (normr \o f) else 0)%E
46+
| +oo%E => (if mu [set: T] > 0 then ess_supr mu (normr \o f) else 0)%E
4747
| -oo%E => 0%E
4848
end.
4949
Canonical locked_Lnorm := Unlockable Lnorm.unlock.
@@ -68,7 +68,7 @@ Lemma Lnorm_ge0 p f : 0 <= 'N_p[f].
6868
Proof.
6969
rewrite unlock; move: p => [r/=|/=|//].
7070
by case: ifPn => // r0; exact: poweR_ge0.
71-
by case: ifPn => // /ess_sup_ge0; apply => t/=.
71+
by case: ifPn => // /ess_sup_ger; apply => t/=.
7272
Qed.
7373

7474
Lemma eq_Lnorm p f g : f =1 g -> 'N_p[f] = 'N_p[g].

theories/measure.v

Lines changed: 0 additions & 18 deletions
Original file line numberDiff line numberDiff line change
@@ -5413,21 +5413,3 @@ Lemma measure_dominates_ae_eq m1 m2 f g E : measurable E ->
54135413
Proof. by move=> mE m21 [A [mA A0 ?]]; exists A; split => //; exact: m21. Qed.
54145414

54155415
End absolute_continuity_lemmas.
5416-
5417-
Section essential_supremum.
5418-
Context d {T : semiRingOfSetsType d} {R : realType}.
5419-
Variable mu : {measure set T -> \bar R}.
5420-
Implicit Types f : T -> R.
5421-
5422-
Definition ess_sup f :=
5423-
ereal_inf (EFin @` [set r | mu (f @^-1` `]r, +oo[) = 0]).
5424-
5425-
Lemma ess_sup_ge0 f : 0 < mu [set: T] -> (forall t, 0 <= f t)%R ->
5426-
0 <= ess_sup f.
5427-
Proof.
5428-
move=> muT f0; apply: lb_ereal_inf => _ /= [r /eqP rf <-]; rewrite leNgt.
5429-
apply/negP => r0; apply/negP : rf; rewrite gt_eqF// (_ : _ @^-1` _ = setT)//.
5430-
by apply/seteqP; split => // x _ /=; rewrite in_itv/= (lt_le_trans _ (f0 x)).
5431-
Qed.
5432-
5433-
End essential_supremum.

0 commit comments

Comments
 (0)