Step * of Lemma ip-line-circle-lemma

rv:InnerProductSpace. ∀r:ℝ. ∀p,q:Point.
  (p q
   (||p|| ≤ r)
   let in
         (r0 ≤ (((r(2) p ⋅ v) r(2) p ⋅ v) r(4) ||v||^2 (||p||^2 r^2)))
         ∧ (||p quadratic1(||v||^2;r(2) p ⋅ v;||p||^2 r^2)*v|| r)
         ∧ (||p quadratic2(||v||^2;r(2) p ⋅ v;||p||^2 r^2)*v|| r))
BY
(Auto THEN Assert ⌜r0 ≤ (p ⋅ p^2 ||q p||^2 (||p||^2 r^2))⌝⋅}

1
.....assertion..... 
1. rv InnerProductSpace
2. : ℝ
3. Point
4. Point
5. q
6. ||p|| ≤ r
⊢ r0 ≤ (p ⋅ p^2 ||q p||^2 (||p||^2 r^2))

2
1. rv InnerProductSpace
2. : ℝ
3. Point
4. Point
5. q
6. ||p|| ≤ r
7. r0 ≤ (p ⋅ p^2 ||q p||^2 (||p||^2 r^2))
⊢ let in
      (r0 ≤ (((r(2) p ⋅ v) r(2) p ⋅ v) r(4) ||v||^2 (||p||^2 r^2)))
      ∧ (||p quadratic1(||v||^2;r(2) p ⋅ v;||p||^2 r^2)*v|| r)
      ∧ (||p quadratic2(||v||^2;r(2) p ⋅ v;||p||^2 r^2)*v|| r)


Latex:


Latex:
\mforall{}rv:InnerProductSpace.  \mforall{}r:\mBbbR{}.  \mforall{}p,q:Point.
    (p  \#  q
    {}\mRightarrow{}  (||p||  \mleq{}  r)
    {}\mRightarrow{}  let  v  =  q  -  p  in
                  (r0  \mleq{}  (((r(2)  *  p  \mcdot{}  v)  *  r(2)  *  p  \mcdot{}  v)  -  r(4)  *  ||v||\^{}2  *  (||p||\^{}2  -  r\^{}2)))
                  \mwedge{}  (||p  +  quadratic1(||v||\^{}2;r(2)  *  p  \mcdot{}  v;||p||\^{}2  -  r\^{}2)*v||  =  r)
                  \mwedge{}  (||p  +  quadratic2(||v||\^{}2;r(2)  *  p  \mcdot{}  v;||p||\^{}2  -  r\^{}2)*v||  =  r))


By


Latex:
(Auto  THEN  Assert  \mkleeneopen{}r0  \mleq{}  (p  \mcdot{}  q  -  p\^{}2  -  ||q  -  p||\^{}2  *  (||p||\^{}2  -  r\^{}2))\mkleeneclose{}\mcdot{})




Home Index