refactor: Linting substrings
This commit is contained in:
parent
cee38b7be8
commit
ac1132c7ca
40 changed files with 133 additions and 132 deletions
|
@ -52,7 +52,7 @@ lemma lineInPlaneCond_perm {S : (PureU1 (n)).LinSols} (hS : LineInPlaneCond S)
|
|||
not_false_eq_true]
|
||||
|
||||
lemma lineInPlaneCond_eq_last' {S : (PureU1 (n.succ.succ)).LinSols} (hS : LineInPlaneCond S)
|
||||
(h : ¬ (S.val ((Fin.last n).castSucc))^2 = (S.val ((Fin.last n).succ))^2 ) :
|
||||
(h : ¬ (S.val ((Fin.last n).castSucc))^2 = (S.val ((Fin.last n).succ))^2) :
|
||||
(2 - n) * S.val (Fin.last (n + 1)) =
|
||||
- (2 - n)* S.val (Fin.castSucc (Fin.last n)) := by
|
||||
erw [sq_eq_sq_iff_eq_or_eq_neg] at h
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue