PhysLean Documentation

PhysLean.Relativity.Lorentz.ComplexVector.Modules

Modules associated with complex Lorentz vectors #

We define the modules underlying complex Lorentz vectors. These definitions are preludes to the definitions of Lorentz.complexContr and Lorentz.complexCo.

The module for contravariant (up-index) complex Lorentz vectors.

Instances For

    The equivalence between ContrℂModule and Fin 1 ⊕ Fin 3 → ℂ.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem Lorentz.ContrℂModule.ext (ψ ψ' : ContrℂModule) (h : ψ.val = ψ'.val) :
      ψ = ψ'
      @[simp]
      theorem Lorentz.ContrℂModule.val_add (ψ ψ' : ContrℂModule) :
      (ψ + ψ').val = ψ.val + ψ'.val
      @[simp]
      theorem Lorentz.ContrℂModule.val_smul (r : ) (ψ : ContrℂModule) :
      (r ψ).val = r ψ.val
      @[simp]
      theorem Lorentz.ContrℂModule.toFin13ℂEquiv_symm_apply_val (a✝ : Fin 1 Fin 3) (a✝¹ : Fin 1 Fin 3) :
      (toFin13ℂEquiv.symm a✝).val a✝¹ = a✝ a✝¹
      @[simp]
      theorem Lorentz.ContrℂModule.toFin13ℂEquiv_apply (a✝ : ContrℂModule) (a✝¹ : Fin 1 Fin 3) :
      toFin13ℂEquiv a✝ a✝¹ = toFin13ℂFun a✝ a✝¹
      @[reducible, inline]

      The underlying element of Fin 1 ⊕ Fin 3 → ℂ of a element in ContrℂModule defined through the linear equivalence toFin13ℂEquiv.

      Equations
      Instances For

        The representation of the Lorentz group on ContrℂModule.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          The module for covariant (up-index) complex Lorentz vectors.

          Instances For

            The equivalence between CoℂModule and Fin 1 ⊕ Fin 3 → ℂ.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              theorem Lorentz.CoℂModule.toFin13ℂEquiv_apply (a✝ : CoℂModule) (a✝¹ : Fin 1 Fin 3) :
              toFin13ℂEquiv a✝ a✝¹ = toFin13ℂFun a✝ a✝¹
              @[simp]
              theorem Lorentz.CoℂModule.toFin13ℂEquiv_symm_apply_val (a✝ : Fin 1 Fin 3) (a✝¹ : Fin 1 Fin 3) :
              (toFin13ℂEquiv.symm a✝).val a✝¹ = a✝ a✝¹
              @[reducible, inline]

              The underlying element of Fin 1 ⊕ Fin 3 → ℂ of a element in CoℂModule defined through the linear equivalence toFin13ℂEquiv.

              Equations
              Instances For

                The representation of the Lorentz group on CoℂModule.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For