Skip to content
Open
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
5 changes: 5 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -106,6 +106,11 @@

- in `lebesgue_integrable.v`:
+ lemma `integrable_norm`
- in `num_topology.v`:
+ lemmas `continuous_rsubmx`, `continuous_lsubmx`

- in `derive.v`:
+ lemmas `differentiable_rsubmx`, `differentiable_lsubmx`

### Changed

Expand Down
16 changes: 15 additions & 1 deletion theories/derive.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
(* mathcomp analysis (c) 2026 Inria and AIST. License: CeCILL-C. *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect ssralg ssrnum matrix interval poly.
From mathcomp Require Import sesquilinear.
Expand Down Expand Up @@ -760,6 +760,20 @@ move=> dfx dgfx; apply: DiffDef; first exact: differentiable_comp.
by rewrite diff_comp // !diff_val.
Qed.

Lemma differentiable_rsubmx m {n1 n2} (f : V -> 'M[R]_(m, n1 + n2)) v :
(forall x, differentiable f x) -> differentiable (rsubmx \o f) v.
Proof.
move=> df; apply: differentiable_comp => //.
exact/linear_differentiable/continuous_rsubmx.
Qed.

Lemma differentiable_lsubmx m {n1 n2} (f : V -> 'M[R]_(m, n1 + n2)) v :
(forall x, differentiable f x) -> differentiable (lsubmx \o f) v.
Proof.
move=> df1; apply: differentiable_comp => //.
exact/linear_differentiable/continuous_lsubmx.
Qed.

Lemma bilinear_schwarz (U V' W' : normedModType R)
(f : {bilinear U -> V' -> W'}) : continuous (fun p => f p.1 p.2) ->
exists2 k, k > 0 & forall u v, `|f u v| <= k * `|u| * `|v|.
Expand Down
2 changes: 1 addition & 1 deletion theories/normedtype_theory/matrix_normedtype.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
(* mathcomp analysis (c) 2026 Inria and AIST. License: CeCILL-C. *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum matrix interval.
From mathcomp Require Import boolp classical_sets interval_inference reals.
Expand Down
6 changes: 5 additions & 1 deletion theories/realfun.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
(* mathcomp analysis (c) 2025 Inria and AIST. License: CeCILL-C. *)
(* mathcomp analysis (c) 2026 Inria and AIST. License: CeCILL-C. *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect finmap ssralg ssrnum ssrint.
From mathcomp Require Import archimedean interval.
Expand Down Expand Up @@ -1880,6 +1880,10 @@ rewrite -[x]sqrtK//; apply: (@is_derive_inverse _ (fun x => x ^+ 2)).
- by rewrite mulf_neq0// gt_eqF// sqrtr_gt0 exprn_gt0// sqrtr_gt0.
Unshelve. all: by end_near. Qed.

Lemma derive_sqrt {K : realType} (r : K) : 0 < r ->
'D_1 Num.sqrt r = (2 * Num.sqrt r)^-1.
Proof. by move=> r0; apply: derive_val; exact: is_derive1_sqrt. Qed.

#[global] Hint Extern 0 (is_derive _ _ (fun _ => (_ _)^-1) _) =>
(eapply is_deriveV; first by []) : typeclass_instances.

Expand Down
3 changes: 2 additions & 1 deletion theories/topology_theory/matrix_topology.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,9 @@
(* mathcomp analysis (c) 2017 Inria and AIST. License: CeCILL-C. *)
(* mathcomp analysis (c) 2026 Inria and AIST. License: CeCILL-C. *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect all_algebra finmap all_classical.
From mathcomp Require Import interval_inference topology_structure.
From mathcomp Require Import uniform_structure pseudometric_structure.

(**md**************************************************************************)
(* # Matrix topology *)
(* ``` *)
Expand Down
20 changes: 18 additions & 2 deletions theories/topology_theory/num_topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,13 +3,13 @@ From HB Require Import structures.
From mathcomp Require Import all_ssreflect all_algebra all_classical.
From mathcomp Require Import interval_inference reals topology_structure.
From mathcomp Require Import uniform_structure pseudometric_structure.
From mathcomp Require Import order_topology.
From mathcomp Require Import order_topology matrix_topology.

(**md**************************************************************************)
(* # Topological notions for numerical types *)
(* *)
(* We endow `numFieldType` with the types of topological notions (accessible *)
(* with `Import numFieldTopology.Exports). *)
(* with `Import numFieldTopology.Exports`). *)
(* *)
(******************************************************************************)

Expand Down Expand Up @@ -378,3 +378,19 @@ have inj_nat_of_rat : injective nat_of_rat.
exact/bij_inj.
by exists (nat_of_rat \o f) => i j Di Dj /inj_nat_of_rat/inj_f; exact.
Qed.

Lemma continuous_rsubmx {R : numFieldType} m {n1 n2} :
continuous (rsubmx : 'M[R]_(m, n1 + n2) -> 'M[R]_(m, n2)).
Proof.
move=> u A /nbhs_ballP[e /= e0 eA].
apply/nbhs_ballP; exists e => //= v [_ uv]; apply: eA; split => // i j.
by apply: (le_lt_trans _ (uv i (rshift n1 j))); rewrite !mxE.
Qed.

Lemma continuous_lsubmx {R : numFieldType} m {n1 n2} :
continuous (lsubmx : 'M[R]_(m, n1 + n2) -> 'M[R]_(m, n1)).
Proof.
move=> u A /nbhs_ballP[e /= e0 eA].
apply/nbhs_ballP; exists e => //= v [_ uv]; apply: eA; split => // i j.
by apply: (le_lt_trans _ (uv i (lshift n2 j))); rewrite !mxE.
Qed.