src/HOL/Library/Code_Real_Approx_By_Float.thy
changeset 54489 03ff4d1e6784
parent 52435 6646bb548c6b
child 60017 b785d6d06430
equal deleted inserted replaced
54488:b60f1fab408c 54489:03ff4d1e6784
   167 lemma [code_unfold del]:
   167 lemma [code_unfold del]:
   168   "numeral k \<equiv> (of_rat (numeral k) :: real)"
   168   "numeral k \<equiv> (of_rat (numeral k) :: real)"
   169   by simp
   169   by simp
   170 
   170 
   171 lemma [code_unfold del]:
   171 lemma [code_unfold del]:
   172   "neg_numeral k \<equiv> (of_rat (neg_numeral k) :: real)"
   172   "- numeral k \<equiv> (of_rat (- numeral k) :: real)"
   173   by simp
   173   by simp
   174 
   174 
   175 hide_const (open) real_of_int
   175 hide_const (open) real_of_int
   176 
   176 
   177 code_printing
   177 code_printing