src/HOL/Hyperreal/HyperBin.ML
changeset 10778 2c6605049646
parent 10751 a81ea5d3dd41
child 10784 27e4d90b35b5
equal deleted inserted replaced
10777:a5a6255748c3 10778:2c6605049646
   168 by Auto_tac;
   168 by Auto_tac;
   169 qed "hypreal_add_number_of_diff2";
   169 qed "hypreal_add_number_of_diff2";
   170 
   170 
   171 Addsimps [hypreal_add_number_of_left, hypreal_mult_number_of_left,
   171 Addsimps [hypreal_add_number_of_left, hypreal_mult_number_of_left,
   172 	  hypreal_add_number_of_diff1, hypreal_add_number_of_diff2]; 
   172 	  hypreal_add_number_of_diff1, hypreal_add_number_of_diff2]; 
   173 
       
   174 
       
   175 (*"neg" is used in rewrite rules for binary comparisons*)
       
   176 Goal "hypreal_of_nat (number_of v :: nat) = \
       
   177 \        (if neg (number_of v) then #0 \
       
   178 \         else (number_of v :: hypreal))";
       
   179 by (simp_tac (simpset() addsimps [hypreal_of_nat_real_of_nat]) 1);
       
   180 qed "hypreal_of_nat_number_of";
       
   181 Addsimps [hypreal_of_nat_number_of];
       
   182 
   173 
   183 
   174 
   184 (**** Simprocs for numeric literals ****)
   175 (**** Simprocs for numeric literals ****)
   185 
   176 
   186 (** Combining of literal coefficients in sums of products **)
   177 (** Combining of literal coefficients in sums of products **)