refactor: Remove double empty lines
This commit is contained in:
parent
ae18a2196d
commit
f03d063c86
60 changed files with 0 additions and 232 deletions
|
@ -120,7 +120,6 @@ lemma boundary_accGrav' (k : Fin n) : accGrav n.succ S =
|
|||
intro i
|
||||
simp
|
||||
|
||||
|
||||
lemma boundary_accGrav'' (k : Fin n) (hk : Boundary S k) :
|
||||
accGrav n.succ S = (2 * ↑↑k + 1 - ↑n) * S (0 : Fin n.succ) := by
|
||||
rw [boundary_accGrav' k]
|
||||
|
@ -165,7 +164,6 @@ lemma not_hasBoundary_grav (hnot : ¬ (HasBoundary S)) :
|
|||
accGrav n.succ S = n.succ * S (0 : Fin n.succ) := by
|
||||
simp [accGrav, ← not_hasBoundry_zero hS hnot]
|
||||
|
||||
|
||||
lemma AFL_hasBoundary (h : A.val (0 : Fin n.succ) ≠ 0) : HasBoundary A.val := by
|
||||
by_contra hn
|
||||
have h0 := not_hasBoundary_grav hA hn
|
||||
|
@ -253,12 +251,10 @@ lemma AFL_even_above (A : (PureU1 (2 * n.succ)).LinSols) (h : ConstAbsSorted A.v
|
|||
rfl
|
||||
exact AFL_even_above' h hA i
|
||||
|
||||
|
||||
end charges
|
||||
|
||||
end ConstAbsSorted
|
||||
|
||||
|
||||
namespace ConstAbs
|
||||
|
||||
theorem boundary_value_odd (S : (PureU1 (2 * n + 1)).LinSols) (hs : ConstAbs S.val) :
|
||||
|
@ -266,7 +262,6 @@ theorem boundary_value_odd (S : (PureU1 (2 * n + 1)).LinSols) (hs : ConstAbs S.v
|
|||
have hS := And.intro (constAbs_sort hs) (sort_sorted S.val)
|
||||
sortAFL_zero S (ConstAbsSorted.AFL_odd (sortAFL S) hS)
|
||||
|
||||
|
||||
theorem boundary_value_even (S : (PureU1 (2 * n.succ)).LinSols) (hs : ConstAbs S.val) :
|
||||
VectorLikeEven S.val := by
|
||||
have hS := And.intro (constAbs_sort hs) (sort_sorted S.val)
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue