Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist authored and mkerjean committed Oct 10, 2024
1 parent b630a5b commit a6da51e
Show file tree
Hide file tree
Showing 4 changed files with 3 additions and 7 deletions.
1 change: 0 additions & 1 deletion theories/charge.v
Original file line number Diff line number Diff line change
Expand Up @@ -91,7 +91,6 @@ Unset Strict Implicit.
Unset Printing Implicit Defensive.

Import Order.TTheory GRing.Theory Num.Def Num.Theory.
Import numFieldTopology.Exports.
Import numFieldNormedType.Exports.

Local Open Scope ring_scope.
Expand Down
7 changes: 3 additions & 4 deletions theories/ftc.v
Original file line number Diff line number Diff line change
Expand Up @@ -24,7 +24,6 @@ Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Import Order.TTheory GRing.Theory Num.Def Num.Theory.
Import numFieldTopology.Exports.
Import numFieldNormedType.Exports.

Local Open Scope classical_set_scope.
Expand All @@ -39,7 +38,7 @@ Implicit Types (f : R -> R) (a : itv_bound R).
Let FTC0 f a : mu.-integrable setT (EFin \o f) ->
let F x := (\int[mu]_(t in [set` Interval a (BRight x)]) f t)%R in
forall x, a < BRight x -> lebesgue_pt f x ->
h^-1 *: (F (h + x) - F x) @[h --> (0:R)%R^'] --> f x.
h^-1 *: (F (h + x) - F x) @[h --> 0%R^'] --> f x.
Proof.
move=> intf F x ax fx.
have locf : locally_integrable setT f.
Expand Down Expand Up @@ -191,7 +190,7 @@ Let FTC0_restrict f a x (u : R) : (x < u)%R ->
mu.-integrable [set` Interval a (BRight u)] (EFin \o f) ->
let F y := (\int[mu]_(t in [set` Interval a (BRight y)]) f t)%R in
a < BRight x -> lebesgue_pt f x ->
h^-1 *: (F (h + x) - F x) @[h --> ((0:R)%R^')] --> f x.
h^-1 *: (F (h + x) - F x) @[h --> (0%R^')] --> f x.
Proof.
move=> xu + F ax fx.
rewrite integrable_mkcond//= (restrict_EFin f) => intf.
Expand Down Expand Up @@ -354,7 +353,7 @@ Unshelve. all: by end_near. Qed.

Lemma parameterized_integral_cvg_left a b (f : R -> R) : a < b ->
mu.-integrable `[a, b] (EFin \o f) ->
int a x f @[x --> a] --> (0:R).
int a x f @[x --> a] --> 0.
Proof.
move=> ab intf; pose fab := f \_ `[a, b].
have intfab : mu.-integrable `[a, b] (EFin \o fab).
Expand Down
1 change: 0 additions & 1 deletion theories/lebesgue_integral.v
Original file line number Diff line number Diff line change
Expand Up @@ -82,7 +82,6 @@ Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Import Order.TTheory GRing.Theory Num.Def Num.Theory.
Import numFieldTopology.Exports.
Import numFieldNormedType.Exports.
From mathcomp Require Import mathcomp_extra.

Expand Down
1 change: 0 additions & 1 deletion theories/lebesgue_measure.v
Original file line number Diff line number Diff line change
Expand Up @@ -61,7 +61,6 @@ Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Import Order.TTheory GRing.Theory Num.Def Num.Theory.
Import numFieldTopology.Exports.
Import numFieldNormedType.Exports.

Local Open Scope classical_set_scope.
Expand Down

0 comments on commit a6da51e

Please sign in to comment.