analysis.calculus.deriv.linear โŸท Mathlib.Analysis.Calculus.Deriv.Linear

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
@@ -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"
 
Diff
@@ -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"
 
Diff
@@ -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
 
Diff
@@ -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
 
Diff
@@ -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
Diff
@@ -27,7 +27,7 @@ derivative, linear map
 
 universe u v w
 
-open Topology Filter
+open scoped Topology Filter
 
 open Filter Asymptotics Set
 

Changes in mathlib4

mathlib3
mathlib4
chore(*): remove empty lines between variable statements (#11418)

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)
Diff
@@ -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
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,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
 
feat: port Analysis.Calculus.Deriv.Linear (#4439)

Dependencies 10 + 675

676 files ported (98.5%)
300730 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