src/HOL/Deriv.thy
changeset 59862 44b3f4fa33ca
parent 59615 fdfdf89a83a6
child 59867 58043346ca64
equal deleted inserted replaced
59860:a979fc5db526 59862:44b3f4fa33ca
   558 
   558 
   559 lemma DERIV_subset: 
   559 lemma DERIV_subset: 
   560   "(f has_field_derivative f') (at x within s) \<Longrightarrow> t \<subseteq> s 
   560   "(f has_field_derivative f') (at x within s) \<Longrightarrow> t \<subseteq> s 
   561    \<Longrightarrow> (f has_field_derivative f') (at x within t)"
   561    \<Longrightarrow> (f has_field_derivative f') (at x within t)"
   562   by (simp add: has_field_derivative_def has_derivative_within_subset)
   562   by (simp add: has_field_derivative_def has_derivative_within_subset)
       
   563 
       
   564 lemma has_field_derivative_at_within:
       
   565     "(f has_field_derivative f') (at x) \<Longrightarrow> (f has_field_derivative f') (at x within s)"
       
   566   using DERIV_subset by blast
   563 
   567 
   564 abbreviation (input)
   568 abbreviation (input)
   565   DERIV :: "('a::real_normed_field \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
   569   DERIV :: "('a::real_normed_field \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
   566   ("(DERIV (_)/ (_)/ :> (_))" [1000, 1000, 60] 60)
   570   ("(DERIV (_)/ (_)/ :> (_))" [1000, 1000, 60] 60)
   567 where
   571 where