src/HOL/Hyperreal/HyperDef.thy
changeset 14341 a09441bd4f1e
parent 14334 6137d24eef79
child 14348 744c868ee0b7
--- a/src/HOL/Hyperreal/HyperDef.thy	Tue Jan 06 10:38:14 2004 +0100
+++ b/src/HOL/Hyperreal/HyperDef.thy	Tue Jan 06 10:40:15 2004 +0100
@@ -474,6 +474,9 @@
   show "0 \<noteq> (1::hypreal)" by (rule hypreal_zero_not_eq_one)
   show "x \<noteq> 0 ==> inverse x * x = 1" by (simp add: hypreal_mult_inverse_left)
   show "y \<noteq> 0 ==> x / y = x * inverse y" by (simp add: hypreal_divide_def)
+  assume eq: "z+x = z+y" 
+    hence "(-z + z) + x = (-z + z) + y" by (simp only: eq hypreal_add_assoc)
+    thus "x = y" by (simp add: hypreal_add_minus_left)
 qed