Skip to content

Commit

Permalink
feat(topology/algebra/monoid): add is_submonoid.mem_nhds_one
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Mar 10, 2019
1 parent 51c31ce commit a756d9e
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions src/topology/algebra/monoid.lean
Expand Up @@ -114,6 +114,11 @@ lemma continuous_finset_prod [topological_space β] {f : γ → β → α} (s :
(∀c∈s, continuous (f c)) → continuous (λa, s.prod (λc, f c a)) :=
continuous_multiset_prod _

@[to_additive is_add_submonoid.mem_nhds_zero]
lemma is_submonoid.mem_nhds_one (β : set α) [is_submonoid β] (oβ : is_open β) :
β ∈ nhds (1 : α) :=
mem_nhds_sets_iff.2 ⟨β, (by refl), oβ, is_submonoid.one_mem _⟩

end

end topological_monoid

0 comments on commit a756d9e

Please sign in to comment.