diff -r e95831757903 -r 67dec4ccaabd src/HOL/Library/Extended_Real.thy --- a/src/HOL/Library/Extended_Real.thy Tue Nov 12 14:24:34 2013 +0100 +++ b/src/HOL/Library/Extended_Real.thy Tue Nov 12 19:28:50 2013 +0100 @@ -156,7 +156,7 @@ subsubsection "Addition" -instantiation ereal :: "{one,comm_monoid_add}" +instantiation ereal :: "{one,comm_monoid_add,zero_neq_one}" begin definition "0 = ereal 0" @@ -197,6 +197,8 @@ by (cases rule: ereal2_cases[of a b]) simp_all show "a + b + c = a + (b + c)" by (cases rule: ereal3_cases[of a b c]) simp_all + show "0 \ (1::ereal)" + by (simp add: one_ereal_def zero_ereal_def) qed end