src/HOL/Hyperreal/Lim.thy
changeset 20635 e95db20977c5
parent 20563 44eda2314aab
child 20653 24cda2c5fd40
equal deleted inserted replaced
20634:45fe31e72391 20635:e95db20977c5
    72        in if P(x, (x+y)/2) then ((x+y)/2, y)
    72        in if P(x, (x+y)/2) then ((x+y)/2, y)
    73                             else (x, (x+y)/2))"
    73                             else (x, (x+y)/2))"
    74 
    74 
    75 
    75 
    76 
    76 
    77 section{*Some Purely Standard Proofs*}
    77 subsection{*Some Purely Standard Proofs*}
    78 
    78 
    79 lemma LIM_eq:
    79 lemma LIM_eq:
    80      "f -- a --> L =
    80      "f -- a --> L =
    81      (\<forall>r>0.\<exists>s>0.\<forall>x. x \<noteq> a & norm (x-a) < s --> norm (f x - L) < r)"
    81      (\<forall>r>0.\<exists>s>0.\<forall>x. x \<noteq> a & norm (x-a) < s --> norm (f x - L) < r)"
    82 by (simp add: LIM_def diff_minus)
    82 by (simp add: LIM_def diff_minus)