analysis.calculus.deriv.linear
โท
Mathlib.Analysis.Calculus.Deriv.Linear
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.
(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)
mathlib commit https://github.com/leanprover-community/mathlib/commit/65a1391a0106c9204fe45bc73a039f056558cb83
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner, Yury Kudryashov
-/
import Analysis.Calculus.Deriv.Basic
-import Analysis.Calculus.Fderiv.Linear
+import Analysis.Calculus.FDeriv.Linear
#align_import analysis.calculus.deriv.linear from "leanprover-community/mathlib"@"f60c6087a7275b72d5db3c5a1d0e19e35a429c0a"
mathlib commit https://github.com/leanprover-community/mathlib/commit/ce64cd319bb6b3e82f31c2d38e79080d377be451
@@ -3,8 +3,8 @@ Copyright (c) 2019 Gabriel Ebner. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner, Yury Kudryashov
-/
-import Mathbin.Analysis.Calculus.Deriv.Basic
-import Mathbin.Analysis.Calculus.Fderiv.Linear
+import Analysis.Calculus.Deriv.Basic
+import Analysis.Calculus.Fderiv.Linear
#align_import analysis.calculus.deriv.linear from "leanprover-community/mathlib"@"f60c6087a7275b72d5db3c5a1d0e19e35a429c0a"
mathlib commit https://github.com/leanprover-community/mathlib/commit/8ea5598db6caeddde6cb734aa179cc2408dbd345
@@ -2,15 +2,12 @@
Copyright (c) 2019 Gabriel Ebner. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner, Yury Kudryashov
-
-! This file was ported from Lean 3 source module analysis.calculus.deriv.linear
-! leanprover-community/mathlib commit f60c6087a7275b72d5db3c5a1d0e19e35a429c0a
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
-/
import Mathbin.Analysis.Calculus.Deriv.Basic
import Mathbin.Analysis.Calculus.Fderiv.Linear
+#align_import analysis.calculus.deriv.linear from "leanprover-community/mathlib"@"f60c6087a7275b72d5db3c5a1d0e19e35a429c0a"
+
/-!
# Derivatives of continuous linear maps from the base field
mathlib commit https://github.com/leanprover-community/mathlib/commit/9fb8964792b4237dac6200193a0d533f1b3f7423
@@ -53,31 +53,43 @@ section ContinuousLinearMap
variable (e : ๐ โL[๐] F)
+#print ContinuousLinearMap.hasDerivAtFilter /-
protected theorem ContinuousLinearMap.hasDerivAtFilter : HasDerivAtFilter e (e 1) x L :=
e.HasFDerivAtFilter.HasDerivAtFilter
#align continuous_linear_map.has_deriv_at_filter ContinuousLinearMap.hasDerivAtFilter
+-/
+#print ContinuousLinearMap.hasStrictDerivAt /-
protected theorem ContinuousLinearMap.hasStrictDerivAt : HasStrictDerivAt e (e 1) x :=
e.HasStrictFDerivAt.HasStrictDerivAt
#align continuous_linear_map.has_strict_deriv_at ContinuousLinearMap.hasStrictDerivAt
+-/
+#print ContinuousLinearMap.hasDerivAt /-
protected theorem ContinuousLinearMap.hasDerivAt : HasDerivAt e (e 1) x :=
e.HasDerivAtFilter
#align continuous_linear_map.has_deriv_at ContinuousLinearMap.hasDerivAt
+-/
+#print ContinuousLinearMap.hasDerivWithinAt /-
protected theorem ContinuousLinearMap.hasDerivWithinAt : HasDerivWithinAt e (e 1) s x :=
e.HasDerivAtFilter
#align continuous_linear_map.has_deriv_within_at ContinuousLinearMap.hasDerivWithinAt
+-/
+#print ContinuousLinearMap.deriv /-
@[simp]
protected theorem ContinuousLinearMap.deriv : deriv e x = e 1 :=
e.HasDerivAt.deriv
#align continuous_linear_map.deriv ContinuousLinearMap.deriv
+-/
+#print ContinuousLinearMap.derivWithin /-
protected theorem ContinuousLinearMap.derivWithin (hxs : UniqueDiffWithinAt ๐ s x) :
derivWithin e s x = e 1 :=
e.HasDerivWithinAt.derivWithin hxs
#align continuous_linear_map.deriv_within ContinuousLinearMap.derivWithin
+-/
end ContinuousLinearMap
@@ -88,31 +100,43 @@ section LinearMap
variable (e : ๐ โโ[๐] F)
+#print LinearMap.hasDerivAtFilter /-
protected theorem LinearMap.hasDerivAtFilter : HasDerivAtFilter e (e 1) x L :=
e.toContinuousLinearMapโ.HasDerivAtFilter
#align linear_map.has_deriv_at_filter LinearMap.hasDerivAtFilter
+-/
+#print LinearMap.hasStrictDerivAt /-
protected theorem LinearMap.hasStrictDerivAt : HasStrictDerivAt e (e 1) x :=
e.toContinuousLinearMapโ.HasStrictDerivAt
#align linear_map.has_strict_deriv_at LinearMap.hasStrictDerivAt
+-/
+#print LinearMap.hasDerivAt /-
protected theorem LinearMap.hasDerivAt : HasDerivAt e (e 1) x :=
e.HasDerivAtFilter
#align linear_map.has_deriv_at LinearMap.hasDerivAt
+-/
+#print LinearMap.hasDerivWithinAt /-
protected theorem LinearMap.hasDerivWithinAt : HasDerivWithinAt e (e 1) s x :=
e.HasDerivAtFilter
#align linear_map.has_deriv_within_at LinearMap.hasDerivWithinAt
+-/
+#print LinearMap.deriv /-
@[simp]
protected theorem LinearMap.deriv : deriv e x = e 1 :=
e.HasDerivAt.deriv
#align linear_map.deriv LinearMap.deriv
+-/
+#print LinearMap.derivWithin /-
protected theorem LinearMap.derivWithin (hxs : UniqueDiffWithinAt ๐ s x) :
derivWithin e s x = e 1 :=
e.HasDerivWithinAt.derivWithin hxs
#align linear_map.deriv_within LinearMap.derivWithin
+-/
end LinearMap
mathlib commit https://github.com/leanprover-community/mathlib/commit/cca40788df1b8755d5baf17ab2f27dacc2e17acb
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner, Yury Kudryashov
! This file was ported from Lean 3 source module analysis.calculus.deriv.linear
-! leanprover-community/mathlib commit 3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe
+! leanprover-community/mathlib commit f60c6087a7275b72d5db3c5a1d0e19e35a429c0a
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
@@ -14,6 +14,9 @@ import Mathbin.Analysis.Calculus.Fderiv.Linear
/-!
# Derivatives of continuous linear maps from the base field
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
In this file we prove that `f : ๐ โL[๐] E` (or `f : ๐ โโ[๐] E`) has derivative `f 1`.
For a more detailed overview of one-dimensional derivatives in mathlib, see the module docstring of
mathlib commit https://github.com/leanprover-community/mathlib/commit/917c3c072e487b3cccdbfeff17e75b40e45f66cb
@@ -27,7 +27,7 @@ derivative, linear map
universe u v w
-open Topology Filter
+open scoped Topology Filter
open Filter Asymptotics Set
mathlib commit https://github.com/leanprover-community/mathlib/commit/917c3c072e487b3cccdbfeff17e75b40e45f66cb
Empty lines were removed by executing the following Python script twice
import os
import re
# Loop through each file in the repository
for dir_path, dirs, files in os.walk('.'):
for filename in files:
if filename.endswith('.lean'):
file_path = os.path.join(dir_path, filename)
# Open the file and read its contents
with open(file_path, 'r') as file:
content = file.read()
# Use a regular expression to replace sequences of "variable" lines separated by empty lines
# with sequences without empty lines
modified_content = re.sub(r'(variable.*\n)\n(variable(?! .* in))', r'\1\2', content)
# Write the modified content back to the file
with open(file_path, 'w') as file:
file.write(modified_content)
@@ -29,15 +29,10 @@ open Topology Filter
open Filter Asymptotics Set
variable {๐ : Type u} [NontriviallyNormedField ๐]
-
variable {F : Type v} [NormedAddCommGroup F] [NormedSpace ๐ F]
-
variable {E : Type w} [NormedAddCommGroup E] [NormedSpace ๐ E]
-
variable {x : ๐}
-
variable {s : Set ๐}
-
variable {L : Filter ๐}
section ContinuousLinearMap
@@ -2,15 +2,12 @@
Copyright (c) 2019 Gabriel Ebner. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Gabriel Ebner, Yury Kudryashov
-
-! This file was ported from Lean 3 source module analysis.calculus.deriv.linear
-! 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.Basic
import Mathlib.Analysis.Calculus.FDeriv.Linear
+#align_import analysis.calculus.deriv.linear from "leanprover-community/mathlib"@"3bce8d800a6f2b8f63fe1e588fd76a9ff4adcebe"
+
/-!
# Derivatives of continuous linear maps from the base field
The unported dependencies are
algebra.order.module
init.core
algebra.order.monoid.cancel.defs
algebra.abs
algebra.group_power.lemmas
init.data.list.basic
algebra.order.monoid.cancel.basic
init.data.list.default
topology.subset_properties
init.logic
The following 1 dependencies have changed in mathlib3 since they were ported, which may complicate porting this file