refactor: Lint

This commit is contained in:
jstoobysmith 2024-08-21 06:45:09 -04:00
parent c0499483a8
commit c2eb4bbe9d
8 changed files with 11 additions and 10 deletions

View file

@ -81,7 +81,7 @@ lemma ud_us_neq_zero_iff_ub_neq_one (V : CKMMatrix) :
zero_pow, add_zero, zero_add, sq_eq_one_iff, false_or, neg_eq_self_iff, one_ne_zero]
have h1 := Complex.abs.nonneg [V]ub
rw [h2] at h1
refine (?_ : ¬ 0 ≤ (-1 : ) ) h1
refine (?_ : ¬ 0 ≤ (-1 : )) h1
simp
lemma normSq_Vud_plus_normSq_Vus_neq_zero_ {V : CKMMatrix} (hb : [V]ud ≠ 0 [V]us ≠ 0) :