src/HOL/Transcendental.thy
changeset 36776 c137ae7673d3
parent 35216 7641e8d831d2
child 36777 be5461582d0f
--- a/src/HOL/Transcendental.thy	Sun May 09 09:39:01 2010 -0700
+++ b/src/HOL/Transcendental.thy	Sun May 09 14:21:44 2010 -0700
@@ -1089,7 +1089,7 @@
 apply (rule_tac x = 1 and y = y in linorder_cases)
 apply (drule order_less_imp_le [THEN lemma_exp_total])
 apply (rule_tac [2] x = 0 in exI)
-apply (frule_tac [3] real_inverse_gt_one)
+apply (frule_tac [3] one_less_inverse)
 apply (drule_tac [4] order_less_imp_le [THEN lemma_exp_total], auto)
 apply (rule_tac x = "-x" in exI)
 apply (simp add: exp_minus)