number_theory.modular_forms.jacobi_theta.manifoldMathlib.NumberTheory.ModularForms.JacobiTheta.Manifold

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)

(last sync)

Changes in mathlib3port

mathlib3
mathlib3port
Diff
@@ -3,7 +3,7 @@ Copyright (c) 2023 David Loeffler. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
 -/
-import NumberTheory.ModularForms.JacobiTheta.Basic
+import NumberTheory.ModularForms.JacobiTheta.OneVariable
 import Analysis.Complex.UpperHalfPlane.Manifold
 
 #align_import number_theory.modular_forms.jacobi_theta.manifold from "leanprover-community/mathlib"@"728ef9dbb281241906f25cbeb30f90d83e0bb451"
Diff
@@ -3,8 +3,8 @@ Copyright (c) 2023 David Loeffler. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
 -/
-import Mathbin.NumberTheory.ModularForms.JacobiTheta.Basic
-import Mathbin.Analysis.Complex.UpperHalfPlane.Manifold
+import NumberTheory.ModularForms.JacobiTheta.Basic
+import Analysis.Complex.UpperHalfPlane.Manifold
 
 #align_import number_theory.modular_forms.jacobi_theta.manifold from "leanprover-community/mathlib"@"728ef9dbb281241906f25cbeb30f90d83e0bb451"
 
Diff
@@ -2,15 +2,12 @@
 Copyright (c) 2023 David Loeffler. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
-
-! This file was ported from Lean 3 source module number_theory.modular_forms.jacobi_theta.manifold
-! leanprover-community/mathlib commit 728ef9dbb281241906f25cbeb30f90d83e0bb451
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathbin.NumberTheory.ModularForms.JacobiTheta.Basic
 import Mathbin.Analysis.Complex.UpperHalfPlane.Manifold
 
+#align_import number_theory.modular_forms.jacobi_theta.manifold from "leanprover-community/mathlib"@"728ef9dbb281241906f25cbeb30f90d83e0bb451"
+
 /-!
 # Manifold differentiability of the Jacobi's theta function
 
Diff
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
 
 ! This file was ported from Lean 3 source module number_theory.modular_forms.jacobi_theta.manifold
-! leanprover-community/mathlib commit 57f9349f2fe19d2de7207e99b0341808d977cdcf
+! leanprover-community/mathlib commit 728ef9dbb281241906f25cbeb30f90d83e0bb451
 ! 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.Complex.UpperHalfPlane.Manifold
 /-!
 # Manifold differentiability of the Jacobi's theta function
 
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
 In this file we reformulate differentiability of the Jacobi's theta function in terms of manifold
 differentiability.
 
Diff
@@ -25,7 +25,9 @@ Prove smoothness (in terms of `smooth`).
 
 open scoped UpperHalfPlane Manifold
 
-theorem mDifferentiable_jacobiTheta : MDifferentiable 𝓘(ℂ) 𝓘(ℂ) (jacobiTheta ∘ coe : ℍ → ℂ) :=
+#print mdifferentiable_jacobiTheta /-
+theorem mdifferentiable_jacobiTheta : MDifferentiable 𝓘(ℂ) 𝓘(ℂ) (jacobiTheta ∘ coe : ℍ → ℂ) :=
   fun τ => (differentiableAt_jacobiTheta τ.2).MDifferentiableAt.comp τ τ.mdifferentiable_coe
-#align mdifferentiable_jacobi_theta mDifferentiable_jacobiTheta
+#align mdifferentiable_jacobi_theta mdifferentiable_jacobiTheta
+-/
 
Diff
@@ -26,6 +26,6 @@ Prove smoothness (in terms of `smooth`).
 open scoped UpperHalfPlane Manifold
 
 theorem mDifferentiable_jacobiTheta : MDifferentiable 𝓘(ℂ) 𝓘(ℂ) (jacobiTheta ∘ coe : ℍ → ℂ) :=
-  fun τ => (differentiableAt_jacobiTheta τ.2).MDifferentiableAt.comp τ τ.mDifferentiable_coe
+  fun τ => (differentiableAt_jacobiTheta τ.2).MDifferentiableAt.comp τ τ.mdifferentiable_coe
 #align mdifferentiable_jacobi_theta mDifferentiable_jacobiTheta
 
Diff
@@ -25,7 +25,7 @@ Prove smoothness (in terms of `smooth`).
 
 open scoped UpperHalfPlane Manifold
 
-theorem mdifferentiable_jacobiTheta : Mdifferentiable 𝓘(ℂ) 𝓘(ℂ) (jacobiTheta ∘ coe : ℍ → ℂ) :=
-  fun τ => (differentiableAt_jacobiTheta τ.2).MdifferentiableAt.comp τ τ.mdifferentiable_coe
-#align mdifferentiable_jacobi_theta mdifferentiable_jacobiTheta
+theorem mDifferentiable_jacobiTheta : MDifferentiable 𝓘(ℂ) 𝓘(ℂ) (jacobiTheta ∘ coe : ℍ → ℂ) :=
+  fun τ => (differentiableAt_jacobiTheta τ.2).MDifferentiableAt.comp τ τ.mDifferentiable_coe
+#align mdifferentiable_jacobi_theta mDifferentiable_jacobiTheta
 

Changes in mathlib4

mathlib3
mathlib4
feat(NumberTheory/ModularForms): two-variable Jacobi theta (#9666)

Add a more general version of the Jacobi theta function with a second variable, and prove the transformation law for this more general function rather than just for the one-variable version. Preparatory to functional equations for Dirichlet L-functions.

Diff
@@ -4,8 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
 -/
 import Mathlib.Analysis.Complex.UpperHalfPlane.Manifold
-import Mathlib.Geometry.Manifold.MFDeriv.SpecificFunctions
-import Mathlib.NumberTheory.ModularForms.JacobiTheta.Basic
+import Mathlib.Geometry.Manifold.MFDeriv.FDeriv
+import Mathlib.NumberTheory.ModularForms.JacobiTheta.OneVariable
 
 #align_import number_theory.modular_forms.jacobi_theta.manifold from "leanprover-community/mathlib"@"57f9349f2fe19d2de7207e99b0341808d977cdcf"
 
refactor(Geometry/Manifold/MFDeriv): split file (#9565)

With about 2200 lines, this is the largest file in Geometry/Manifolds.

Diff
@@ -3,8 +3,9 @@ Copyright (c) 2023 David Loeffler. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
 -/
-import Mathlib.NumberTheory.ModularForms.JacobiTheta.Basic
 import Mathlib.Analysis.Complex.UpperHalfPlane.Manifold
+import Mathlib.Geometry.Manifold.MFDeriv.SpecificFunctions
+import Mathlib.NumberTheory.ModularForms.JacobiTheta.Basic
 
 #align_import number_theory.modular_forms.jacobi_theta.manifold from "leanprover-community/mathlib"@"57f9349f2fe19d2de7207e99b0341808d977cdcf"
 
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) 2023 David Loeffler. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: David Loeffler
-
-! This file was ported from Lean 3 source module number_theory.modular_forms.jacobi_theta.manifold
-! leanprover-community/mathlib commit 57f9349f2fe19d2de7207e99b0341808d977cdcf
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathlib.NumberTheory.ModularForms.JacobiTheta.Basic
 import Mathlib.Analysis.Complex.UpperHalfPlane.Manifold
 
+#align_import number_theory.modular_forms.jacobi_theta.manifold from "leanprover-community/mathlib"@"57f9349f2fe19d2de7207e99b0341808d977cdcf"
+
 /-!
 # Manifold differentiability of the Jacobi theta function
 
feat: port NumberTheory.ModularForms.JacobiTheta.Manifold (#5670)

Dependencies 12 + 1199

1200 files ported (99.0%)
537675 lines ported (99.0%)
Show graph

The unported dependencies are

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