refactor: Remove double empty lines
This commit is contained in:
parent
ae18a2196d
commit
f03d063c86
60 changed files with 0 additions and 232 deletions
|
@ -17,12 +17,10 @@ related by phase shifts.
|
|||
The notation `[V]ud` etc can be used for the elements of a CKM matrix, and
|
||||
`[V]ud|us` etc for the ratios of elements.
|
||||
|
||||
|
||||
-/
|
||||
|
||||
open Matrix Complex
|
||||
|
||||
|
||||
noncomputable section
|
||||
|
||||
/-- Given three real numbers `a b c` the complex matrix with `exp (I * a)` etc on the
|
||||
|
@ -107,7 +105,6 @@ lemma phaseShiftRelation_trans {U V W : unitaryGroup (Fin 3) ℂ} :
|
|||
rw [phaseShiftMatrix_mul]
|
||||
rw [add_comm k e, add_comm l f, add_comm m g]
|
||||
|
||||
|
||||
lemma phaseShiftRelation_equiv : Equivalence PhaseShiftRelation where
|
||||
refl := phaseShiftRelation_refl
|
||||
symm := phaseShiftRelation_symm
|
||||
|
@ -270,7 +267,6 @@ lemma tb (V : CKMMatrix) (a b c d e f : ℝ) :
|
|||
|
||||
end phaseShiftApply
|
||||
|
||||
|
||||
/-- The aboslute value of the `(i,j)`th element of `V`. -/
|
||||
@[simp]
|
||||
def VAbs' (V : unitaryGroup (Fin 3) ℂ) (i j : Fin 3) : ℝ := Complex.abs (V i j)
|
||||
|
@ -341,11 +337,9 @@ abbrev VtsAbs := VAbs 2 1
|
|||
@[simp]
|
||||
abbrev VtbAbs := VAbs 2 2
|
||||
|
||||
|
||||
namespace CKMMatrix
|
||||
open ComplexConjugate
|
||||
|
||||
|
||||
section ratios
|
||||
|
||||
/-- The ratio of the `ub` and `ud` elements of a CKM matrix. -/
|
||||
|
@ -394,7 +388,6 @@ lemma Rcscb_mul_cb {V : CKMMatrix} (h : [V]cb ≠ 0): [V]cs = Rcscb V * [V]cb :=
|
|||
|
||||
end ratios
|
||||
|
||||
|
||||
end CKMMatrix
|
||||
|
||||
end
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue