src/HOL/Deriv.thy
changeset 68644 242d298526a3
parent 68638 87d1bff264df
child 69020 4f94e262976d
equal deleted inserted replaced
68638:87d1bff264df 68644:242d298526a3
  1084 lemmas has_derivative_floor[derivative_intros] =
  1084 lemmas has_derivative_floor[derivative_intros] =
  1085   floor_has_real_derivative[THEN DERIV_compose_FDERIV]
  1085   floor_has_real_derivative[THEN DERIV_compose_FDERIV]
  1086 
  1086 
  1087 text \<open>Caratheodory formulation of derivative at a point\<close>
  1087 text \<open>Caratheodory formulation of derivative at a point\<close>
  1088 
  1088 
  1089 lemma CARAT_DERIV: (*FIXME: SUPERSEDED BY THE ONE IN Deriv.thy. But still used by NSA/HDeriv.thy*)
  1089 lemma CARAT_DERIV:
  1090   "(DERIV f x :> l) \<longleftrightarrow> (\<exists>g. (\<forall>z. f z - f x = g z * (z - x)) \<and> isCont g x \<and> g x = l)"
  1090   "(DERIV f x :> l) \<longleftrightarrow> (\<exists>g. (\<forall>z. f z - f x = g z * (z - x)) \<and> isCont g x \<and> g x = l)"
  1091   (is "?lhs = ?rhs")
  1091   (is "?lhs = ?rhs")
  1092 proof
  1092 proof
  1093   assume ?lhs
  1093   assume ?lhs
  1094   show "\<exists>g. (\<forall>z. f z - f x = g z * (z - x)) \<and> isCont g x \<and> g x = l"
  1094   show "\<exists>g. (\<forall>z. f z - f x = g z * (z - x)) \<and> isCont g x \<and> g x = l"
  1101     show "?g x = l"
  1101     show "?g x = l"
  1102       by simp
  1102       by simp
  1103   qed
  1103   qed
  1104 next
  1104 next
  1105   assume ?rhs
  1105   assume ?rhs
  1106   then obtain g where "(\<forall>z. f z - f x = g z * (z - x))" and "isCont g x" and "g x = l"
       
  1107     by blast
       
  1108   then show ?lhs
  1106   then show ?lhs
  1109     by (auto simp add: isCont_iff DERIV_def cong: LIM_cong)
  1107     by (auto simp add: isCont_iff DERIV_def cong: LIM_cong)
  1110 qed
  1108 qed
  1111 
  1109 
  1112 
  1110