src/HOL/Real/RealVector.thy
changeset 21404 eb85850d3eb7
parent 21210 c17fd2df4e9e
child 21809 4b93e949ac33
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    39 
    39 
    40 consts
    40 consts
    41   scaleR :: "real \<Rightarrow> 'a \<Rightarrow> 'a::scaleR" (infixr "*#" 75)
    41   scaleR :: "real \<Rightarrow> 'a \<Rightarrow> 'a::scaleR" (infixr "*#" 75)
    42 
    42 
    43 abbreviation
    43 abbreviation
    44   divideR :: "'a \<Rightarrow> real \<Rightarrow> 'a::scaleR" (infixl "'/#" 70)
    44   divideR :: "'a \<Rightarrow> real \<Rightarrow> 'a::scaleR" (infixl "'/#" 70) where
    45   "x /# r == inverse r *# x"
    45   "x /# r == inverse r *# x"
    46 
    46 
    47 notation (xsymbols)
    47 notation (xsymbols)
    48   scaleR (infixr "*\<^sub>R" 75)
    48   scaleR (infixr "*\<^sub>R" 75) and
    49   divideR (infixl "'/\<^sub>R" 70)
    49   divideR (infixl "'/\<^sub>R" 70)
    50 
    50 
    51 instance real :: scaleR ..
    51 instance real :: scaleR ..
    52 
    52 
    53 defs (overloaded)
    53 defs (overloaded)
   173 
   173 
   174 subsection {* Embedding of the Reals into any @{text real_algebra_1}:
   174 subsection {* Embedding of the Reals into any @{text real_algebra_1}:
   175 @{term of_real} *}
   175 @{term of_real} *}
   176 
   176 
   177 definition
   177 definition
   178   of_real :: "real \<Rightarrow> 'a::real_algebra_1"
   178   of_real :: "real \<Rightarrow> 'a::real_algebra_1" where
   179   "of_real r = r *# 1"
   179   "of_real r = r *# 1"
   180 
   180 
   181 lemma scaleR_conv_of_real: "r *# x = of_real r * x"
   181 lemma scaleR_conv_of_real: "r *# x = of_real r * x"
   182 by (simp add: of_real_def)
   182 by (simp add: of_real_def)
   183 
   183 
   248 
   248 
   249 
   249 
   250 subsection {* The Set of Real Numbers *}
   250 subsection {* The Set of Real Numbers *}
   251 
   251 
   252 definition
   252 definition
   253   Reals :: "'a::real_algebra_1 set"
   253   Reals :: "'a::real_algebra_1 set" where
   254   "Reals \<equiv> range of_real"
   254   "Reals \<equiv> range of_real"
   255 
   255 
   256 notation (xsymbols)
   256 notation (xsymbols)
   257   Reals  ("\<real>")
   257   Reals  ("\<real>")
   258 
   258