src/HOL/Analysis/Linear_Algebra.thy
changeset 68607 67bb59e49834
parent 68224 1f7308050349
child 68901 4824cc40f42e
--- a/src/HOL/Analysis/Linear_Algebra.thy	Mon Jul 09 21:55:40 2018 +0100
+++ b/src/HOL/Analysis/Linear_Algebra.thy	Tue Jul 10 09:38:35 2018 +0200
@@ -377,11 +377,11 @@
 subsection \<open>Archimedean properties and useful consequences\<close>
 
 text\<open>Bernoulli's inequality\<close>
-proposition%important Bernoulli_inequality:
+proposition Bernoulli_inequality:
   fixes x :: real
   assumes "-1 \<le> x"
     shows "1 + n * x \<le> (1 + x) ^ n"
-proof%unimportant (induct n)
+proof (induct n)
   case 0
   then show ?case by simp
 next