Skip to content

Commit

Permalink
chore(analysis/topology/continuity): locally_compact_space is Prop
Browse files Browse the repository at this point in the history
  • Loading branch information
johoelzl committed Oct 17, 2018
1 parent bac655d commit ea962a7
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion analysis/topology/continuity.lean
Expand Up @@ -713,7 +713,7 @@ section locally_compact
Hausdorff spaces but not in general. This one is the precise condition on X needed for the
evaluation `map C(X, Y) × X → Y` to be continuous for all `Y` when `C(X, Y)` is given the
compact-open topology. -/
class locally_compact_space (α : Type*) [topological_space α] :=
class locally_compact_space (α : Type*) [topological_space α] : Prop :=
(local_compact_nhds : ∀ (x : α) (n ∈ (nhds x).sets), ∃ s ∈ (nhds x).sets, s ⊆ n ∧ compact s)

lemma locally_compact_of_compact_nhds [topological_space α] [t2_space α]
Expand Down

0 comments on commit ea962a7

Please sign in to comment.