src/HOL/Library/Extended_Real.thy
changeset 45769 2d5b1af2426a
parent 45236 ac4a2a66707d
child 45934 9321cd2572fe
--- a/src/HOL/Library/Extended_Real.thy	Mon Dec 05 14:47:01 2011 +0100
+++ b/src/HOL/Library/Extended_Real.thy	Mon Dec 05 17:33:57 2011 +0100
@@ -59,7 +59,7 @@
 
 declare [[coercion "ereal :: real \<Rightarrow> ereal"]]
 declare [[coercion "ereal_of_enat :: enat \<Rightarrow> ereal"]]
-declare [[coercion "(\<lambda>n. ereal (of_nat n)) :: nat \<Rightarrow> ereal"]]
+declare [[coercion "(\<lambda>n. ereal (real n)) :: nat \<Rightarrow> ereal"]]
 
 lemma ereal_uminus_uminus[simp]:
   fixes a :: ereal shows "- (- a) = a"