analysis.calculus.diff_cont_on_cl ⟷ Mathlib.Analysis.Calculus.DiffContOnCl

This file has been ported!

Changes since the initial port

The following section lists changes to this file in mathlib3 and mathlib4 that occured after the initial port. Most recent changes are shown first. Hovering over a commit will show all commits associated with the same mathlib3 commit.

Changes in mathlib3

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(last sync)

Changes in mathlib3port

mathlib3
mathlib3port
Diff
@@ -3,7 +3,7 @@ Copyright (c) 2022 Yury G. Kudryashov. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Yury G. Kudryashov
 -/
-import Mathbin.Analysis.Calculus.Deriv.Inv
+import Analysis.Calculus.Deriv.Inv
 
 #align_import analysis.calculus.diff_cont_on_cl from "leanprover-community/mathlib"@"61b5e2755ccb464b68d05a9acf891ae04992d09d"
 
Diff
@@ -104,10 +104,10 @@ protected theorem differentiableAt (h : DiffContOnCl π•œ f s) (hs : IsOpen s) (
 #align diff_cont_on_cl.differentiable_at DiffContOnCl.differentiableAt
 -/
 
-#print DiffContOnCl.differentiable_at' /-
-theorem differentiable_at' (h : DiffContOnCl π•œ f s) (hx : s ∈ 𝓝 x) : DifferentiableAt π•œ f x :=
+#print DiffContOnCl.differentiableAt' /-
+theorem differentiableAt' (h : DiffContOnCl π•œ f s) (hx : s ∈ 𝓝 x) : DifferentiableAt π•œ f x :=
   h.DifferentiableOn.DifferentiableAt hx
-#align diff_cont_on_cl.differentiable_at' DiffContOnCl.differentiable_at'
+#align diff_cont_on_cl.differentiable_at' DiffContOnCl.differentiableAt'
 -/
 
 #print DiffContOnCl.mono /-
Diff
@@ -2,14 +2,11 @@
 Copyright (c) 2022 Yury G. Kudryashov. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Yury G. Kudryashov
-
-! This file was ported from Lean 3 source module analysis.calculus.diff_cont_on_cl
-! leanprover-community/mathlib commit 61b5e2755ccb464b68d05a9acf891ae04992d09d
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathbin.Analysis.Calculus.Deriv.Inv
 
+#align_import analysis.calculus.diff_cont_on_cl from "leanprover-community/mathlib"@"61b5e2755ccb464b68d05a9acf891ae04992d09d"
+
 /-!
 # Functions differentiable on a domain and continuous on its closure
 
Diff
@@ -42,33 +42,46 @@ structure DiffContOnCl (f : E β†’ F) (s : Set E) : Prop where
 
 variable {π•œ}
 
+#print DifferentiableOn.diffContOnCl /-
 theorem DifferentiableOn.diffContOnCl (h : DifferentiableOn π•œ f (closure s)) : DiffContOnCl π•œ f s :=
   ⟨h.mono subset_closure, h.ContinuousOn⟩
 #align differentiable_on.diff_cont_on_cl DifferentiableOn.diffContOnCl
+-/
 
+#print Differentiable.diffContOnCl /-
 theorem Differentiable.diffContOnCl (h : Differentiable π•œ f) : DiffContOnCl π•œ f s :=
   ⟨h.DifferentiableOn, h.Continuous.ContinuousOn⟩
 #align differentiable.diff_cont_on_cl Differentiable.diffContOnCl
+-/
 
+#print IsClosed.diffContOnCl_iff /-
 theorem IsClosed.diffContOnCl_iff (hs : IsClosed s) : DiffContOnCl π•œ f s ↔ DifferentiableOn π•œ f s :=
   ⟨fun h => h.DifferentiableOn, fun h => ⟨h, hs.closure_eq.symm β–Έ h.ContinuousOn⟩⟩
 #align is_closed.diff_cont_on_cl_iff IsClosed.diffContOnCl_iff
+-/
 
+#print diffContOnCl_univ /-
 theorem diffContOnCl_univ : DiffContOnCl π•œ f univ ↔ Differentiable π•œ f :=
   isClosed_univ.diffContOnCl_iff.trans differentiableOn_univ
 #align diff_cont_on_cl_univ diffContOnCl_univ
+-/
 
+#print diffContOnCl_const /-
 theorem diffContOnCl_const {c : F} : DiffContOnCl π•œ (fun x : E => c) s :=
   ⟨differentiableOn_const c, continuousOn_const⟩
 #align diff_cont_on_cl_const diffContOnCl_const
+-/
 
 namespace DiffContOnCl
 
+#print DiffContOnCl.comp /-
 theorem comp {g : G β†’ E} {t : Set G} (hf : DiffContOnCl π•œ f s) (hg : DiffContOnCl π•œ g t)
     (h : MapsTo g t s) : DiffContOnCl π•œ (f ∘ g) t :=
   ⟨hf.1.comp hg.1 h, hf.2.comp hg.2 <| h.closure_of_continuousOn hg.2⟩
 #align diff_cont_on_cl.comp DiffContOnCl.comp
+-/
 
+#print DiffContOnCl.continuousOn_ball /-
 theorem continuousOn_ball [NormedSpace ℝ E] {x : E} {r : ℝ} (h : DiffContOnCl π•œ f (ball x r)) :
     ContinuousOn f (closedBall x r) :=
   by
@@ -78,84 +91,119 @@ theorem continuousOn_ball [NormedSpace ℝ E] {x : E} {r : ℝ} (h : DiffContOnC
   Β· rw [← closure_ball x hr]
     exact h.continuous_on
 #align diff_cont_on_cl.continuous_on_ball DiffContOnCl.continuousOn_ball
+-/
 
+#print DiffContOnCl.mk_ball /-
 theorem mk_ball {x : E} {r : ℝ} (hd : DifferentiableOn π•œ f (ball x r))
     (hc : ContinuousOn f (closedBall x r)) : DiffContOnCl π•œ f (ball x r) :=
   ⟨hd, hc.mono <| closure_ball_subset_closedBall⟩
 #align diff_cont_on_cl.mk_ball DiffContOnCl.mk_ball
+-/
 
+#print DiffContOnCl.differentiableAt /-
 protected theorem differentiableAt (h : DiffContOnCl π•œ f s) (hs : IsOpen s) (hx : x ∈ s) :
     DifferentiableAt π•œ f x :=
   h.DifferentiableOn.DifferentiableAt <| hs.mem_nhds hx
 #align diff_cont_on_cl.differentiable_at DiffContOnCl.differentiableAt
+-/
 
+#print DiffContOnCl.differentiable_at' /-
 theorem differentiable_at' (h : DiffContOnCl π•œ f s) (hx : s ∈ 𝓝 x) : DifferentiableAt π•œ f x :=
   h.DifferentiableOn.DifferentiableAt hx
 #align diff_cont_on_cl.differentiable_at' DiffContOnCl.differentiable_at'
+-/
 
+#print DiffContOnCl.mono /-
 protected theorem mono (h : DiffContOnCl π•œ f s) (ht : t βŠ† s) : DiffContOnCl π•œ f t :=
   ⟨h.DifferentiableOn.mono ht, h.ContinuousOn.mono (closure_mono ht)⟩
 #align diff_cont_on_cl.mono DiffContOnCl.mono
+-/
 
+#print DiffContOnCl.add /-
 theorem add (hf : DiffContOnCl π•œ f s) (hg : DiffContOnCl π•œ g s) : DiffContOnCl π•œ (f + g) s :=
   ⟨hf.1.add hg.1, hf.2.add hg.2⟩
 #align diff_cont_on_cl.add DiffContOnCl.add
+-/
 
+#print DiffContOnCl.add_const /-
 theorem add_const (hf : DiffContOnCl π•œ f s) (c : F) : DiffContOnCl π•œ (fun x => f x + c) s :=
   hf.add diffContOnCl_const
 #align diff_cont_on_cl.add_const DiffContOnCl.add_const
+-/
 
+#print DiffContOnCl.const_add /-
 theorem const_add (hf : DiffContOnCl π•œ f s) (c : F) : DiffContOnCl π•œ (fun x => c + f x) s :=
   diffContOnCl_const.add hf
 #align diff_cont_on_cl.const_add DiffContOnCl.const_add
+-/
 
+#print DiffContOnCl.neg /-
 theorem neg (hf : DiffContOnCl π•œ f s) : DiffContOnCl π•œ (-f) s :=
   ⟨hf.1.neg, hf.2.neg⟩
 #align diff_cont_on_cl.neg DiffContOnCl.neg
+-/
 
+#print DiffContOnCl.sub /-
 theorem sub (hf : DiffContOnCl π•œ f s) (hg : DiffContOnCl π•œ g s) : DiffContOnCl π•œ (f - g) s :=
   ⟨hf.1.sub hg.1, hf.2.sub hg.2⟩
 #align diff_cont_on_cl.sub DiffContOnCl.sub
+-/
 
+#print DiffContOnCl.sub_const /-
 theorem sub_const (hf : DiffContOnCl π•œ f s) (c : F) : DiffContOnCl π•œ (fun x => f x - c) s :=
   hf.sub diffContOnCl_const
 #align diff_cont_on_cl.sub_const DiffContOnCl.sub_const
+-/
 
+#print DiffContOnCl.const_sub /-
 theorem const_sub (hf : DiffContOnCl π•œ f s) (c : F) : DiffContOnCl π•œ (fun x => c - f x) s :=
   diffContOnCl_const.sub hf
 #align diff_cont_on_cl.const_sub DiffContOnCl.const_sub
+-/
 
+#print DiffContOnCl.const_smul /-
 theorem const_smul {R : Type _} [Semiring R] [Module R F] [SMulCommClass π•œ R F]
     [ContinuousConstSMul R F] (hf : DiffContOnCl π•œ f s) (c : R) : DiffContOnCl π•œ (c β€’ f) s :=
   ⟨hf.1.const_smul c, hf.2.const_smul c⟩
 #align diff_cont_on_cl.const_smul DiffContOnCl.const_smul
+-/
 
+#print DiffContOnCl.smul /-
 theorem smul {π•œ' : Type _} [NontriviallyNormedField π•œ'] [NormedAlgebra π•œ π•œ'] [NormedSpace π•œ' F]
     [IsScalarTower π•œ π•œ' F] {c : E β†’ π•œ'} {f : E β†’ F} {s : Set E} (hc : DiffContOnCl π•œ c s)
     (hf : DiffContOnCl π•œ f s) : DiffContOnCl π•œ (fun x => c x β€’ f x) s :=
   ⟨hc.1.smul hf.1, hc.2.smul hf.2⟩
 #align diff_cont_on_cl.smul DiffContOnCl.smul
+-/
 
+#print DiffContOnCl.smul_const /-
 theorem smul_const {π•œ' : Type _} [NontriviallyNormedField π•œ'] [NormedAlgebra π•œ π•œ']
     [NormedSpace π•œ' F] [IsScalarTower π•œ π•œ' F] {c : E β†’ π•œ'} {s : Set E} (hc : DiffContOnCl π•œ c s)
     (y : F) : DiffContOnCl π•œ (fun x => c x β€’ y) s :=
   hc.smul diffContOnCl_const
 #align diff_cont_on_cl.smul_const DiffContOnCl.smul_const
+-/
 
+#print DiffContOnCl.inv /-
 theorem inv {f : E β†’ π•œ} (hf : DiffContOnCl π•œ f s) (hβ‚€ : βˆ€ x ∈ closure s, f x β‰  0) :
     DiffContOnCl π•œ f⁻¹ s :=
   ⟨differentiableOn_inv.comp hf.1 fun x hx => hβ‚€ _ (subset_closure hx), hf.2.invβ‚€ hβ‚€βŸ©
 #align diff_cont_on_cl.inv DiffContOnCl.inv
+-/
 
 end DiffContOnCl
 
+#print Differentiable.comp_diffContOnCl /-
 theorem Differentiable.comp_diffContOnCl {g : G β†’ E} {t : Set G} (hf : Differentiable π•œ f)
     (hg : DiffContOnCl π•œ g t) : DiffContOnCl π•œ (f ∘ g) t :=
   hf.DiffContOnCl.comp hg (mapsTo_image _ _)
 #align differentiable.comp_diff_cont_on_cl Differentiable.comp_diffContOnCl
+-/
 
+#print DifferentiableOn.diffContOnCl_ball /-
 theorem DifferentiableOn.diffContOnCl_ball {U : Set E} {c : E} {R : ℝ} (hf : DifferentiableOn π•œ f U)
     (hc : closedBall c R βŠ† U) : DiffContOnCl π•œ f (ball c R) :=
   DiffContOnCl.mk_ball (hf.mono (ball_subset_closedBall.trans hc)) (hf.ContinuousOn.mono hc)
 #align differentiable_on.diff_cont_on_cl_ball DifferentiableOn.diffContOnCl_ball
+-/
 
Diff
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Yury G. Kudryashov
 
 ! This file was ported from Lean 3 source module analysis.calculus.diff_cont_on_cl
-! leanprover-community/mathlib commit 3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe
+! leanprover-community/mathlib commit 61b5e2755ccb464b68d05a9acf891ae04992d09d
 ! Please do not edit these lines, except to modify the commit id
 ! if you have ported upstream changes.
 -/
@@ -13,6 +13,9 @@ import Mathbin.Analysis.Calculus.Deriv.Inv
 /-!
 # Functions differentiable on a domain and continuous on its closure
 
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
 Many theorems in complex analysis assume that a function is complex differentiable on a domain and
 is continuous on its closure. In this file we define a predicate `diff_cont_on_cl` that expresses
 this property and prove basic facts about this predicate.
@@ -27,6 +30,7 @@ variable (π•œ : Type _) {E F G : Type _} [NontriviallyNormedField π•œ] [Normed
   [NormedAddCommGroup F] [NormedSpace π•œ E] [NormedSpace π•œ F] [NormedAddCommGroup G]
   [NormedSpace π•œ G] {f g : E β†’ F} {s t : Set E} {x : E}
 
+#print DiffContOnCl /-
 /-- A predicate saying that a function is differentiable on a set and is continuous on its
 closure. This is a common assumption in complex analysis. -/
 @[protect_proj]
@@ -34,6 +38,7 @@ structure DiffContOnCl (f : E β†’ F) (s : Set E) : Prop where
   DifferentiableOn : DifferentiableOn π•œ f s
   ContinuousOn : ContinuousOn f (closure s)
 #align diff_cont_on_cl DiffContOnCl
+-/
 
 variable {π•œ}
 
Diff
@@ -21,7 +21,7 @@ this property and prove basic facts about this predicate.
 
 open Set Filter Metric
 
-open Topology
+open scoped Topology
 
 variable (π•œ : Type _) {E F G : Type _} [NontriviallyNormedField π•œ] [NormedAddCommGroup E]
   [NormedAddCommGroup F] [NormedSpace π•œ E] [NormedSpace π•œ F] [NormedAddCommGroup G]
Diff
@@ -4,11 +4,11 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Yury G. Kudryashov
 
 ! This file was ported from Lean 3 source module analysis.calculus.diff_cont_on_cl
-! leanprover-community/mathlib commit f2ce6086713c78a7f880485f7917ea547a215982
+! leanprover-community/mathlib commit 3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe
 ! Please do not edit these lines, except to modify the commit id
 ! if you have ported upstream changes.
 -/
-import Mathbin.Analysis.Calculus.Deriv
+import Mathbin.Analysis.Calculus.Deriv.Inv
 
 /-!
 # Functions differentiable on a domain and continuous on its closure

Changes in mathlib4

mathlib3
mathlib4
chore(NormedSpace/Basic): move some theorems to NormedSpace.Real (#10206)

This way we don't switch between general normed spaces and real normed spaces back and forth throughout the file.

Diff
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Yury G. Kudryashov
 -/
 import Mathlib.Analysis.Calculus.Deriv.Inv
+import Mathlib.Analysis.NormedSpace.Real
 
 #align_import analysis.calculus.diff_cont_on_cl from "leanprover-community/mathlib"@"3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe"
 
chore: banish Type _ and Sort _ (#6499)

We remove all possible occurences of Type _ and Sort _ in favor of Type* and Sort*.

This has nice performance benefits.

Diff
@@ -20,7 +20,7 @@ open Set Filter Metric
 
 open scoped Topology
 
-variable (π•œ : Type _) {E F G : Type _} [NontriviallyNormedField π•œ] [NormedAddCommGroup E]
+variable (π•œ : Type*) {E F G : Type*} [NontriviallyNormedField π•œ] [NormedAddCommGroup E]
   [NormedAddCommGroup F] [NormedSpace π•œ E] [NormedSpace π•œ F] [NormedAddCommGroup G]
   [NormedSpace π•œ G] {f g : E β†’ F} {s t : Set E} {x : E}
 
@@ -115,18 +115,18 @@ theorem const_sub (hf : DiffContOnCl π•œ f s) (c : F) : DiffContOnCl π•œ (fun
   diffContOnCl_const.sub hf
 #align diff_cont_on_cl.const_sub DiffContOnCl.const_sub
 
-theorem const_smul {R : Type _} [Semiring R] [Module R F] [SMulCommClass π•œ R F]
+theorem const_smul {R : Type*} [Semiring R] [Module R F] [SMulCommClass π•œ R F]
     [ContinuousConstSMul R F] (hf : DiffContOnCl π•œ f s) (c : R) : DiffContOnCl π•œ (c β€’ f) s :=
   ⟨hf.1.const_smul c, hf.2.const_smul c⟩
 #align diff_cont_on_cl.const_smul DiffContOnCl.const_smul
 
-theorem smul {π•œ' : Type _} [NontriviallyNormedField π•œ'] [NormedAlgebra π•œ π•œ'] [NormedSpace π•œ' F]
+theorem smul {π•œ' : Type*} [NontriviallyNormedField π•œ'] [NormedAlgebra π•œ π•œ'] [NormedSpace π•œ' F]
     [IsScalarTower π•œ π•œ' F] {c : E β†’ π•œ'} {f : E β†’ F} {s : Set E} (hc : DiffContOnCl π•œ c s)
     (hf : DiffContOnCl π•œ f s) : DiffContOnCl π•œ (fun x => c x β€’ f x) s :=
   ⟨hc.1.smul hf.1, hc.2.smul hf.2⟩
 #align diff_cont_on_cl.smul DiffContOnCl.smul
 
-theorem smul_const {π•œ' : Type _} [NontriviallyNormedField π•œ'] [NormedAlgebra π•œ π•œ']
+theorem smul_const {π•œ' : Type*} [NontriviallyNormedField π•œ'] [NormedAlgebra π•œ π•œ']
     [NormedSpace π•œ' F] [IsScalarTower π•œ π•œ' F] {c : E β†’ π•œ'} {s : Set E} (hc : DiffContOnCl π•œ c s)
     (y : F) : DiffContOnCl π•œ (fun x => c x β€’ y) s :=
   hc.smul diffContOnCl_const
chore: tidy various files (#6382)
Diff
@@ -79,9 +79,9 @@ protected theorem differentiableAt (h : DiffContOnCl π•œ f s) (hs : IsOpen s) (
   h.differentiableOn.differentiableAt <| hs.mem_nhds hx
 #align diff_cont_on_cl.differentiable_at DiffContOnCl.differentiableAt
 
-theorem differentiable_at' (h : DiffContOnCl π•œ f s) (hx : s ∈ 𝓝 x) : DifferentiableAt π•œ f x :=
+theorem differentiableAt' (h : DiffContOnCl π•œ f s) (hx : s ∈ 𝓝 x) : DifferentiableAt π•œ f x :=
   h.differentiableOn.differentiableAt hx
-#align diff_cont_on_cl.differentiable_at' DiffContOnCl.differentiable_at'
+#align diff_cont_on_cl.differentiable_at' DiffContOnCl.differentiableAt'
 
 protected theorem mono (h : DiffContOnCl π•œ f s) (ht : t βŠ† s) : DiffContOnCl π•œ f t :=
   ⟨h.differentiableOn.mono ht, h.continuousOn.mono (closure_mono ht)⟩
chore: script to replace headers with #align_import statements (#5979)

Open in Gitpod

Co-authored-by: Eric Wieser <wieser.eric@gmail.com> Co-authored-by: Scott Morrison <scott.morrison@gmail.com>

Diff
@@ -2,14 +2,11 @@
 Copyright (c) 2022 Yury G. Kudryashov. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Yury G. Kudryashov
-
-! This file was ported from Lean 3 source module analysis.calculus.diff_cont_on_cl
-! leanprover-community/mathlib commit 3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathlib.Analysis.Calculus.Deriv.Inv
 
+#align_import analysis.calculus.diff_cont_on_cl from "leanprover-community/mathlib"@"3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe"
+
 /-!
 # Functions differentiable on a domain and continuous on its closure
 
feat: port Analysis.Complex.CauchyIntegral (#4880)
Diff
@@ -30,8 +30,8 @@ variable (π•œ : Type _) {E F G : Type _} [NontriviallyNormedField π•œ] [Normed
 /-- A predicate saying that a function is differentiable on a set and is continuous on its
 closure. This is a common assumption in complex analysis. -/
 structure DiffContOnCl (f : E β†’ F) (s : Set E) : Prop where
-  protected DifferentiableOn : DifferentiableOn π•œ f s
-  protected ContinuousOn : ContinuousOn f (closure s)
+  protected differentiableOn : DifferentiableOn π•œ f s
+  protected continuousOn : ContinuousOn f (closure s)
 #align diff_cont_on_cl DiffContOnCl
 
 variable {π•œ}
@@ -45,7 +45,7 @@ theorem Differentiable.diffContOnCl (h : Differentiable π•œ f) : DiffContOnCl 
 #align differentiable.diff_cont_on_cl Differentiable.diffContOnCl
 
 theorem IsClosed.diffContOnCl_iff (hs : IsClosed s) : DiffContOnCl π•œ f s ↔ DifferentiableOn π•œ f s :=
-  ⟨fun h => h.DifferentiableOn, fun h => ⟨h, hs.closure_eq.symm β–Έ h.continuousOn⟩⟩
+  ⟨fun h => h.differentiableOn, fun h => ⟨h, hs.closure_eq.symm β–Έ h.continuousOn⟩⟩
 #align is_closed.diff_cont_on_cl_iff IsClosed.diffContOnCl_iff
 
 theorem diffContOnCl_univ : DiffContOnCl π•œ f univ ↔ Differentiable π•œ f :=
@@ -69,7 +69,7 @@ theorem continuousOn_ball [NormedSpace ℝ E] {x : E} {r : ℝ} (h : DiffContOnC
   Β· rw [closedBall_zero]
     exact continuousOn_singleton f x
   Β· rw [← closure_ball x hr]
-    exact h.ContinuousOn
+    exact h.continuousOn
 #align diff_cont_on_cl.continuous_on_ball DiffContOnCl.continuousOn_ball
 
 theorem mk_ball {x : E} {r : ℝ} (hd : DifferentiableOn π•œ f (ball x r))
@@ -79,15 +79,15 @@ theorem mk_ball {x : E} {r : ℝ} (hd : DifferentiableOn π•œ f (ball x r))
 
 protected theorem differentiableAt (h : DiffContOnCl π•œ f s) (hs : IsOpen s) (hx : x ∈ s) :
     DifferentiableAt π•œ f x :=
-  h.DifferentiableOn.differentiableAt <| hs.mem_nhds hx
+  h.differentiableOn.differentiableAt <| hs.mem_nhds hx
 #align diff_cont_on_cl.differentiable_at DiffContOnCl.differentiableAt
 
 theorem differentiable_at' (h : DiffContOnCl π•œ f s) (hx : s ∈ 𝓝 x) : DifferentiableAt π•œ f x :=
-  h.DifferentiableOn.differentiableAt hx
+  h.differentiableOn.differentiableAt hx
 #align diff_cont_on_cl.differentiable_at' DiffContOnCl.differentiable_at'
 
 protected theorem mono (h : DiffContOnCl π•œ f s) (ht : t βŠ† s) : DiffContOnCl π•œ f t :=
-  ⟨h.DifferentiableOn.mono ht, h.ContinuousOn.mono (closure_mono ht)⟩
+  ⟨h.differentiableOn.mono ht, h.continuousOn.mono (closure_mono ht)⟩
 #align diff_cont_on_cl.mono DiffContOnCl.mono
 
 theorem add (hf : DiffContOnCl π•œ f s) (hg : DiffContOnCl π•œ g s) : DiffContOnCl π•œ (f + g) s :=
feat: port Analysis.Calculus.DiffContOnCl (#4492)

Dependencies 10 + 684

685 files ported (98.6%)
303678 lines ported (98.3%)
Show graph

The unported dependencies are

The following 1 dependencies have changed in mathlib3 since they were ported, which may complicate porting this file