Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist committed Jan 2, 2024
1 parent 5ab5c36 commit 7b68f4f
Showing 1 changed file with 10 additions and 2 deletions.
12 changes: 10 additions & 2 deletions theories/topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -2088,6 +2088,8 @@ Next Obligation. done. Qed.

End TopologyOfFilter.

(** Topology defined by open sets *)

Section TopologyOfOpen.

Variable (T : Type) (op : set T -> Prop).
Expand Down Expand Up @@ -2551,6 +2553,8 @@ Qed.

End Weak_Topology.

(** Supremum of a family of topologies *)

Section Sup_Topology.

Variable (T : pointedType) (I : Type) (Tc : I -> Topological.class_of T).
Expand Down Expand Up @@ -2598,6 +2602,8 @@ Definition product_topologicalType :=

End Product_Topology.

(** deleted neighborhood *)

Definition dnbhs {T : topologicalType} (x : T) :=
within (fun y => y != x) (nbhs x).
Notation "x ^'" := (dnbhs x) : classical_set_scope.
Expand Down Expand Up @@ -5266,7 +5272,9 @@ rewrite /= -[leRHS]invrK lef_pinv ?posrE ?invr_gt0// -natr1.
by rewrite natr_absz ger0_norm ?floor_ge0 ?invr_ge0// 1?ltW// lt_succ_floor.
Qed.

(* Specific pseudoMetric spaces *)
(** Specific pseudoMetric spaces *)

(** matrices *)
Section matrix_PseudoMetric.
Variables (m n : nat) (R : numDomainType) (T : pseudoMetricType R).
Implicit Types x y : 'M[T]_(m, n).
Expand Down Expand Up @@ -5303,7 +5311,7 @@ Canonical matrix_pseudoMetricType :=
PseudoMetricType 'M[T]_(m, n) matrix_pseudoMetricType_mixin.
End matrix_PseudoMetric.

(* product of two pseudoMetric spaces *)
(** product of two pseudoMetric spaces *)
Section prod_PseudoMetric.
Context {R : numDomainType} {U V : pseudoMetricType R}.
Implicit Types (x y : U * V).
Expand Down

0 comments on commit 7b68f4f

Please sign in to comment.