src/HOL/Complex/NSCA.thy
changeset 20686 e3d2b881ed0f
parent 20563 44eda2314aab
child 20724 a1a8ba09e0ea
equal deleted inserted replaced
20685:fee8c75e3b5d 20686:e3d2b881ed0f
   110 apply (auto intro: SReal_dense simp add: SReal_hcmod_SComplex)
   110 apply (auto intro: SReal_dense simp add: SReal_hcmod_SComplex)
   111 done
   111 done
   112 
   112 
   113 lemma SComplex_hcmod_SReal: 
   113 lemma SComplex_hcmod_SReal: 
   114       "z \<in> SComplex ==> hcmod z \<in> Reals"
   114       "z \<in> SComplex ==> hcmod z \<in> Reals"
   115 by (auto simp add: SComplex_def SReal_def hcmod_def)
   115 by (auto simp add: SComplex_def)
   116 
   116 
   117 lemma SComplex_zero [simp]: "0 \<in> SComplex"
   117 lemma SComplex_zero [simp]: "0 \<in> SComplex"
   118 by (simp add: SComplex_def)
   118 by (simp add: SComplex_def)
   119 
   119 
   120 lemma SComplex_one [simp]: "1 \<in> SComplex"
   120 lemma SComplex_one [simp]: "1 \<in> SComplex"