src/HOL/Nonstandard_Analysis/Star.thy
changeset 67613 ce654b0e6d69
parent 64435 c93b0e6131c3
child 70218 e48c0b5897a6
equal deleted inserted replaced
67610:4939494ed791 67613:ce654b0e6d69
   229 
   229 
   230 lemma starfun_inverse2: "\<And>x. inverse (( *f* f) x) = ( *f* (\<lambda>x. inverse (f x))) x"
   230 lemma starfun_inverse2: "\<And>x. inverse (( *f* f) x) = ( *f* (\<lambda>x. inverse (f x))) x"
   231   by transfer (rule refl)
   231   by transfer (rule refl)
   232 
   232 
   233 text \<open>General lemma/theorem needed for proofs in elementary topology of the reals.\<close>
   233 text \<open>General lemma/theorem needed for proofs in elementary topology of the reals.\<close>
   234 lemma starfun_mem_starset: "\<And>x. ( *f* f) x : *s* A \<Longrightarrow> x \<in> *s* {x. f x \<in> A}"
   234 lemma starfun_mem_starset: "\<And>x. ( *f* f) x \<in> *s* A \<Longrightarrow> x \<in> *s* {x. f x \<in> A}"
   235   by transfer simp
   235   by transfer simp
   236 
   236 
   237 text \<open>Alternative definition for \<open>hrabs\<close> with \<open>rabs\<close> function applied
   237 text \<open>Alternative definition for \<open>hrabs\<close> with \<open>rabs\<close> function applied
   238   entrywise to equivalence class representative.
   238   entrywise to equivalence class representative.
   239   This is easily proved using @{thm [source] starfun} and ns extension thm.\<close>
   239   This is easily proved using @{thm [source] starfun} and ns extension thm.\<close>