src/HOL/Cardinals/Wellorder_Relation.thy
changeset 55102 761e40ce91bc
parent 55056 b5c94200d081
child 55173 5556470a02b7
--- a/src/HOL/Cardinals/Wellorder_Relation.thy	Wed Jan 22 09:45:30 2014 +0100
+++ b/src/HOL/Cardinals/Wellorder_Relation.thy	Wed Jan 22 10:13:40 2014 +0100
@@ -29,7 +29,7 @@
 using TOTALS by auto
 
 
-subsection {* Well-founded induction and recursion adapted to non-strict well-order relations  *}
+subsection {* Well-founded induction and recursion adapted to non-strict well-order relations *}
 
 lemma worec_unique_fixpoint:
 assumes ADM: "adm_wo H" and fp: "f = H f"
@@ -60,7 +60,7 @@
 qed
 
 
-subsubsection{* Properties of minim *}
+subsubsection {* Properties of minim *}
 
 lemma minim_Under:
 "\<lbrakk>B \<le> Field r; B \<noteq> {}\<rbrakk> \<Longrightarrow> minim B \<in> Under B"
@@ -166,7 +166,7 @@
 qed
 
 
-subsubsection{* Properties of supr *}
+subsubsection {* Properties of supr *}
 
 lemma supr_Above:
 assumes SUB: "B \<le> Field r" and ABOVE: "Above B \<noteq> {}"
@@ -287,7 +287,7 @@
 qed
 
 
-subsubsection{* Properties of successor *}
+subsubsection {* Properties of successor *}
 
 lemma suc_least:
 "\<lbrakk>B \<le> Field r; a \<in> Field r; (\<And> b. b \<in> B \<Longrightarrow> a \<noteq> b \<and> (b,a) \<in> r)\<rbrakk>
@@ -454,7 +454,7 @@
 by(unfold Union_eq, auto)
 
 
-subsubsection{* Other properties *}
+subsubsection {* Other properties *}
 
 lemma Trans_Under_regressive:
 assumes NE: "A \<noteq> {}" and SUB: "A \<le> Field r"