Skip to content
Merged
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
43 changes: 22 additions & 21 deletions theories/function_spaces.v
Original file line number Diff line number Diff line change
Expand Up @@ -109,7 +109,7 @@ Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.

Obligation Tactic := idtac.
Local Obligation Tactic := idtac.

Import Order.TTheory GRing.Theory Num.Theory.
Local Open Scope classical_set_scope.
Expand Down Expand Up @@ -152,13 +152,13 @@ HB.instance Definition _ (U : Type) (T : U -> uniformType) :=
Uniform.copy (forall x : U, T x) (prod_topology T).

HB.instance Definition _ (U T : topologicalType) :=
Topological.copy
(continuousType U T)
Topological.copy
(continuousType U T)
(weak_topology (id : continuousType U T -> (U -> T))).

HB.instance Definition _ (U : topologicalType) (T : uniformType) :=
Uniform.copy
(continuousType U T)
Uniform.copy
(continuousType U T)
(weak_topology (id : continuousType U T -> (U -> T))).

End ArrowAsProduct.
Expand Down Expand Up @@ -222,9 +222,9 @@ Lemma tychonoff (I : eqType) (T : I -> topologicalType)
(forall i, compact (A i)) ->
compact [set f : forall i, T i | forall i, A i (f i)].
Proof.
case: (pselect ([set f : forall i, T i | forall i, A i (f i)] == set0)).
move/eqP => -> _; exact: compact0.
case/negP/set0P=> a0 Aa0 Aco; rewrite compact_ultra => F FU FA.
have [-> _|] := eqVneq [set f : forall i, T i | forall i, A i (f i)] set0.
exact: compact0.
case/set0P => a0 Aa0 Aco; rewrite compact_ultra => F FU FA.
set subst_coord := fun (i : I) (pi : T i) (f : forall x : I, T x) (j : I) =>
if eqP is ReflectT e then ecast i (T i) (esym e) pi else f j.
have subst_coordT i pi f : subst_coord i pi f i = pi.
Expand All @@ -244,12 +244,12 @@ have pFA i : pF i (A i).
move=> Aipi; have [f Af] := filter_ex FA.
exists (subst_coord i pi f); last exact: subst_coordT.
move=> j; have [<-{j}|] := eqVneq i j; first by rewrite subst_coordT.
by move=> /subst_coordN ->; apply: Af.
by move=> /subst_coordN ->; exact: Af.
have cvpFA i : A i `&` [set p | pF i --> p] !=set0.
by rewrite -ultra_cvg_clusterE; apply: Aco.
exists (fun i => xget (a0 i) (A i `&` [set p | pF i --> p])).
split=> [i|]; first by have /(xgetPex (a0 i)) [] := cvpFA i.
apply/cvg_sup => i; apply/cvg_image=> //.
apply/cvg_sup => i; apply/cvg_image=> //.
by have /(xgetPex (a0 i)) [] := cvpFA i.
Qed.

Expand Down Expand Up @@ -423,11 +423,9 @@ Qed.

End product_embeddings.

Global Instance prod_topology_filter (U : Type) (T : U -> ptopologicalType) (f : prod_topology T) :
ProperFilter (nbhs f).
Proof.
exact: nbhs_pfilter.
Qed.
Global Instance prod_topology_filter (U : Type) (T : U -> ptopologicalType)
(f : prod_topology T) : ProperFilter (nbhs f).
Proof. exact: nbhs_pfilter. Qed.

End product_spaces.

Expand Down Expand Up @@ -514,8 +512,11 @@ Unshelve. all: by end_near. Qed.
HB.instance Definition _ := Uniform_isComplete.Build
(arrow_uniform_type T U) fun_complete.

HB.instance Definition _ (R : numFieldType) :=
Uniform_isComplete.Build (arrow_uniform_type T U) cauchy_cvg.
(*HB.instance Definition _ (R : numFieldType) :=
Uniform_isComplete.Build (arrow_uniform_type T U) cauchy_cvg.*)
(* NB: commented out because
Warning: HB: no new instance is generated [HB.no-new-instance,HB,elpi,default]
*)

End fun_Complete.

Expand Down Expand Up @@ -554,13 +555,13 @@ HB.instance Definition _ (U : choiceType) (R : numFieldType)
PseudoMetric.copy (U -> V) (arrow_uniform_type U V).

HB.instance Definition _ (U : topologicalType) (T : uniformType) :=
Uniform.copy
(continuousType U T)
Uniform.copy
(continuousType U T)
(weak_topology (id : continuousType U T -> (U -> T))).

HB.instance Definition _ (U : topologicalType) (R : realType)
HB.instance Definition _ (U : topologicalType) (R : realType)
(T : pseudoMetricType R) :=
PseudoMetric.on
PseudoMetric.on
(weak_topology (id : continuousType U T -> (U -> T))).

End ArrowAsUniformType.
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -65,8 +65,7 @@ Proof. by []. Qed.

End simple_fun_raw_integral.

#[global] Hint Extern 0 (is_true (0 <= (_ : {measure set _ -> \bar _}) _)%E) =>
solve [apply: measure_ge0] : core.
#[global] Hint Extern 0 (is_true (0 <= _)) => solve [apply: measure_ge0] : core.

Section sintegral_lemmas.
Context d (T : sigmaRingType d) (R : realType).
Expand Down
1 change: 0 additions & 1 deletion theories/realfun.v
Original file line number Diff line number Diff line change
Expand Up @@ -38,7 +38,6 @@ From mathcomp Require Import normedtype derive sequences real_interval.
(* total_variation a b f == the sup over all variations of f from a to b *)
(* neg_tv a f x == the decreasing component of f *)
(* pos_tv a f x == the increasing component of f *)
(* *)
(* ``` *)
(* *)
(* Limit superior and inferior for functions: *)
Expand Down
7 changes: 0 additions & 7 deletions theories/topology_theory/matrix_topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -53,13 +53,6 @@ HB.instance Definition _ := Nbhs_isNbhsTopological.Build 'M[T]_(m, n)

End matrix_Topology.

Section matrix_PointedTopology.
Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I'm assuming this does not need an entry in the changelog

Copy link
Member Author

@affeldt-aist affeldt-aist May 1, 2025

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Yes because it was duplicating code that is anyway inaccessible for the user since it is code automatically generated by HB.

Variables (m n : nat) (T : pointedType).
Implicit Types M : 'M[T]_(m, n).
HB.instance Definition _ := Pointed.on 'M[T]_(m, n).

End matrix_PointedTopology.

Section matrix_Uniform.
Local Open Scope relation_scope.
Variables (m n : nat) (T : uniformType).
Expand Down
8 changes: 4 additions & 4 deletions theories/topology_theory/num_topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -109,12 +109,12 @@ by apply: contra_not_neq AsupA => <-.
Qed.

Lemma right_bounded_interior (R : realType) (X : set R) :
has_ubound X -> X^° `<=` [set r | r < sup X].
has_ubound X -> X° `<=` [set r | r < sup X].
Proof.
move=> uX r Xr; rewrite /mkset ltNge; apply/negP.
rewrite le_eqVlt => /orP[/eqP supXr|]; last first.
by apply/negP; rewrite -leNgt sup_ubound//; exact: interior_subset.
suff : ~ X^° (sup X) by rewrite supXr.
suff : ~ X° (sup X) by rewrite supXr.
case/nbhs_ballP => _/posnumP[e] supXeX.
have [f XsupXf] : exists f : {posnum R}, X (sup X + f%:num).
exists (e%:num / 2)%:pos; apply supXeX; rewrite /ball /= opprD addNKr normrN.
Expand All @@ -124,12 +124,12 @@ by apply/negP; rewrite -ltNge; rewrite ltrDl.
Qed.

Lemma left_bounded_interior (R : realType) (X : set R) :
has_lbound X -> X^° `<=` [set r | inf X < r].
has_lbound X -> X° `<=` [set r | inf X < r].
Proof.
move=> lX r Xr; rewrite /mkset ltNge; apply/negP.
rewrite le_eqVlt => /orP[/eqP rinfX|]; last first.
by apply/negP; rewrite -leNgt inf_lbound//; exact: interior_subset.
suff : ~ X^° (inf X) by rewrite -rinfX.
suff : ~ X° (inf X) by rewrite -rinfX.
case/nbhs_ballP => _/posnumP[e] supXeX.
have [f XsupXf] : exists f : {posnum R}, X (inf X - f%:num).
exists (e%:num / 2)%:pos; apply supXeX; rewrite /ball /= opprB addrC subrK.
Expand Down
Loading