src/HOL/Library/Extended_Real.thy
changeset 67727 ce3e87a51488
parent 67685 bdff8bf0a75b
child 68095 4fa3e63ecc7e
equal deleted inserted replaced
67726:0cd2fd0c2dcf 67727:ce3e87a51488
  4295     by eventually_elim auto
  4295     by eventually_elim auto
  4296   ultimately show ?thesis
  4296   ultimately show ?thesis
  4297     by (simp add: x' y' cong: filterlim_cong)
  4297     by (simp add: x' y' cong: filterlim_cong)
  4298 qed
  4298 qed
  4299 
  4299 
       
  4300 lemma continuous_on_diff_ereal:
       
  4301   "continuous_on A f \<Longrightarrow> continuous_on A g \<Longrightarrow> (\<And>x. x \<in> A \<Longrightarrow> \<bar>f x\<bar> \<noteq> \<infinity>) \<Longrightarrow> (\<And>x. x \<in> A \<Longrightarrow> \<bar>g x\<bar> \<noteq> \<infinity>) \<Longrightarrow> continuous_on A (\<lambda>z. f z - g z::ereal)"
       
  4302   apply (auto simp: continuous_on_def)
       
  4303   apply (intro tendsto_diff_ereal)
       
  4304   apply metis+
       
  4305   done
       
  4306 
       
  4307 
  4300 subsubsection \<open>Tests for code generator\<close>
  4308 subsubsection \<open>Tests for code generator\<close>
  4301 
  4309 
  4302 text \<open>A small list of simple arithmetic expressions.\<close>
  4310 text \<open>A small list of simple arithmetic expressions.\<close>
  4303 
  4311 
  4304 value "- \<infinity> :: ereal"
  4312 value "- \<infinity> :: ereal"