Skip to content

Commit

Permalink
more splitting or topology
Browse files Browse the repository at this point in the history
  • Loading branch information
zstone1 committed Oct 4, 2024
1 parent 7dfb606 commit aa9c91f
Show file tree
Hide file tree
Showing 7 changed files with 1,070 additions and 999 deletions.
1 change: 1 addition & 0 deletions _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -27,6 +27,7 @@ theories/reals.v
theories/landau.v
theories/Rstruct.v
theories/topology.v
theories/separation_axioms.v
theories/function_spaces.v
theories/cantor.v
theories/prodnormedzmodule.v
Expand Down
1 change: 1 addition & 0 deletions theories/cantor.v
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,7 @@ From mathcomp Require Import finmap.
From mathcomp Require Import mathcomp_extra boolp classical_sets functions.
From mathcomp Require Import cardinality.
From mathcomp Require Import reals signed topology function_spaces.
From mathcomp Require Import separation_axioms.
From HB Require Import structures.

(**md**************************************************************************)
Expand Down
1 change: 1 addition & 0 deletions theories/derive.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@ From HB Require Import structures.
From mathcomp Require Import all_ssreflect ssralg ssrnum matrix interval.
From mathcomp Require Import mathcomp_extra boolp classical_sets functions.
Require Import reals signed topology prodnormedzmodule normedtype landau forms.
Require Import separation_axioms.

(**md**************************************************************************)
(* # Differentiation *)
Expand Down
4 changes: 2 additions & 2 deletions theories/function_spaces.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ From HB Require Import structures.
From mathcomp Require Import all_ssreflect all_algebra finmap generic_quotient.
From mathcomp Require Import boolp classical_sets functions.
From mathcomp Require Import cardinality mathcomp_extra fsbigop.
Require Import reals signed topology.
Require Import reals signed topology separation_axioms.

(**md**************************************************************************)
(* # The topology of functions spaces *)
Expand Down Expand Up @@ -1421,7 +1421,7 @@ Lemma continuous_uncurry (f : U -> V -> W) :
Proof.
move=> lcV hsdf ctsf cf; apply: continuous_uncurry_regular => //.
move=> v; have [B] := @lcV v I; rewrite withinET => Bv [cptB clB].
by move=> z; exact: (@compact_regular V hsdf v B).
by move=> z; exact: (compact_regular _ cptB).
Qed.

Lemma curry_continuous (f : (U * V)%type -> W) : continuous f -> @regular_space U ->
Expand Down
2 changes: 2 additions & 0 deletions theories/normedtype.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,8 @@ From mathcomp Require Import boolp classical_sets functions.
From mathcomp Require Import archimedean.
From mathcomp Require Import cardinality set_interval Rstruct.
Require Import ereal reals signed topology prodnormedzmodule function_spaces.
Require Import separation_axioms.
Require Export separation_axioms.

(**md**************************************************************************)
(* # Norm-related Notions *)
Expand Down
Loading

0 comments on commit aa9c91f

Please sign in to comment.