Zulip Chat Archive
Stream: Is there code for X?
Topic: is_closed_prod
Ashvni Narayanan (Jun 12 2021 at 11:58):
My goal is to show that the product of clopen sets is clopen. As a supporting statement, I need the following :
lemma is_closed_prod {α β : Type*} [topological_space α] [topological_space β] {s : set α}
{t : set β} (h : is_closed s ∧ is_closed t) : is_closed (set.prod s t) :=
Is this already in mathlib? Thank you!
Sebastien Gouezel (Jun 12 2021 at 12:04):
It's called is_closed.prod
, to make sure that dot notation works fine. I found it using regexp search for is_closed.*prod
in vscode
Eric Wieser (Jun 12 2021 at 12:18):
Lemmas will almost never take P ∧ Q
as an assumption unless they live in the and
namespace (eg docs#and.elim), which probably thwarted your search
Ashvni Narayanan (Jun 12 2021 at 13:15):
Thank you!
Last updated: Dec 20 2023 at 11:08 UTC