src/HOL/ex/Landau.thy
changeset 36809 354b15d5b4ca
parent 36635 080b755377c0
child 39198 f967a16dfcdd
--- a/src/HOL/ex/Landau.thy	Tue May 11 08:29:42 2010 +0200
+++ b/src/HOL/ex/Landau.thy	Tue May 11 08:29:42 2010 +0200
@@ -8,8 +8,8 @@
 begin
 
 text {*
-  We establish a preorder releation @{text "\<lesssim>"} on functions
-  from @{text "\<nat>"} to @{text "\<nat>"} such that @{text "f \<lesssim> g \<longleftrightarrow> f \<in> O(g)"}.
+  We establish a preorder releation @{text "\<lesssim>"} on functions from
+  @{text "\<nat>"} to @{text "\<nat>"} such that @{text "f \<lesssim> g \<longleftrightarrow> f \<in> O(g)"}.
 *}
 
 subsection {* Auxiliary *}
@@ -175,12 +175,12 @@
 
 text {*
   We would like to show (or refute) that @{text "f \<prec> g \<longleftrightarrow> f \<in> o(g)"},
-  i.e.~@{prop "f \<prec> g \<longleftrightarrow> (\<forall>c. \<exists>n. \<forall>m>n. f m < Suc c * g m)"} but did not manage to
-  do so.
+  i.e.~@{prop "f \<prec> g \<longleftrightarrow> (\<forall>c. \<exists>n. \<forall>m>n. f m < Suc c * g m)"} but did not
+  manage to do so.
 *}
 
 
-subsection {* Assert that @{text "\<lesssim>"} is ineed a preorder *}
+subsection {* Assert that @{text "\<lesssim>"} is indeed a preorder *}
 
 interpretation fun_order: preorder_equiv less_eq_fun less_fun
   where "preorder_equiv.equiv less_eq_fun = equiv_fun"