Skip to content

Commit

Permalink
chore: rename Pcontinuous to PContinuous (#4428)
Browse files Browse the repository at this point in the history
ref #4354
  • Loading branch information
urkud committed May 28, 2023
1 parent e258549 commit 3ff6ded
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Topology/Basic.lean
Expand Up @@ -25,7 +25,7 @@ the notion of cluster point of a sequence `u` is `MapClusterPt x atTop u`.
For topological spaces `α` and `β`, a function `f : α → β` and a point `a : α`,
`ContinuousAt f a` means `f` is continuous at `a`, and global continuity is
`Continuous f`. There is also a version of continuity `Pcontinuous` for
`Continuous f`. There is also a version of continuity `PContinuous` for
partially defined functions.
## Notation
Expand Down
10 changes: 5 additions & 5 deletions Mathlib/Topology/Partial.lean
Expand Up @@ -15,7 +15,7 @@ import Mathlib.Order.Filter.Partial
# Partial functions and topological spaces
In this file we prove properties of `Filter.Ptendsto` etc in topological spaces. We also introduce
`Pcontinuous`, a version of `Continuous` for partially defined functions.
`PContinuous`, a version of `Continuous` for partially defined functions.
-/


Expand Down Expand Up @@ -53,16 +53,16 @@ theorem ptendsto'_nhds {f : β →. α} {l : Filter β} {a : α} :
variable [TopologicalSpace β]

/-- Continuity of a partial function -/
def Pcontinuous (f : α →. β) :=
def PContinuous (f : α →. β) :=
∀ s, IsOpen s → IsOpen (f.preimage s)
#align pcontinuous Pcontinuous
#align pcontinuous PContinuous

theorem open_dom_of_pcontinuous {f : α →. β} (h : Pcontinuous f) : IsOpen f.Dom := by
theorem open_dom_of_pcontinuous {f : α →. β} (h : PContinuous f) : IsOpen f.Dom := by
rw [← PFun.preimage_univ]; exact h _ isOpen_univ
#align open_dom_of_pcontinuous open_dom_of_pcontinuous

theorem pcontinuous_iff' {f : α →. β} :
Pcontinuous f ↔ ∀ {x y} (h : y ∈ f x), Ptendsto' f (𝓝 x) (𝓝 y) := by
PContinuous f ↔ ∀ {x y} (h : y ∈ f x), Ptendsto' f (𝓝 x) (𝓝 y) := by
constructor
· intro h x y h'
simp only [ptendsto'_def, mem_nhds_iff]
Expand Down

0 comments on commit 3ff6ded

Please sign in to comment.