Documentation

Mathlib.Analysis.Complex.UpperHalfPlane.FunctionsBoundedAtInfty

Bounded at infinity #

For complex valued functions on the upper half plane, this file defines the filter UpperHalfPlane.atImInfty required for defining when functions are bounded at infinity and zero at infinity. Both of which are relevant for defining modular forms.

Filter for approaching i∞.

Equations
Instances For

    A function f : ℍ → α is bounded at infinity if it is bounded along atImInfty.

    Equations
    Instances For

      A function f : ℍ → α is zero at infinity it is zero along atImInfty.

      Equations
      Instances For

        Module of functions that are zero at infinity.

        Equations
        Instances For
          theorem UpperHalfPlane.bounded_mem (f : UpperHalfPlane) :
          UpperHalfPlane.IsBoundedAtImInfty f ∃ (M : ) (A : ), ∀ (z : UpperHalfPlane), A z.imComplex.abs (f z) M
          theorem UpperHalfPlane.zero_at_im_infty (f : UpperHalfPlane) :
          UpperHalfPlane.IsZeroAtImInfty f ∀ (ε : ), 0 < ε∃ (A : ), ∀ (z : UpperHalfPlane), A z.imComplex.abs (f z) ε