equal
deleted
inserted
replaced
917 show ?thesis by simp |
917 show ?thesis by simp |
918 next |
918 next |
919 assume notless: "~ (0 < x)" |
919 assume notless: "~ (0 < x)" |
920 have "~ (1 < inverse x)" |
920 have "~ (1 < inverse x)" |
921 proof |
921 proof |
922 assume "1 < inverse x" |
922 assume *: "1 < inverse x" |
923 also with notless have "... \<le> 0" by simp |
923 also from notless and * have "... \<le> 0" by simp |
924 also have "... < 1" by (rule zero_less_one) |
924 also have "... < 1" by (rule zero_less_one) |
925 finally show False by auto |
925 finally show False by auto |
926 qed |
926 qed |
927 with notless show ?thesis by simp |
927 with notless show ?thesis by simp |
928 qed |
928 qed |