src/HOL/BNF_Wellorder_Relation.thy
changeset 55173 5556470a02b7
parent 55101 57c875e488bd
child 58889 5b7a9633cfa8
--- a/src/HOL/BNF_Wellorder_Relation.thy	Thu Jan 30 01:03:55 2014 +0100
+++ b/src/HOL/BNF_Wellorder_Relation.thy	Thu Jan 30 12:27:42 2014 +0100
@@ -34,6 +34,8 @@
 abbreviation aboveS where "aboveS \<equiv> Order_Relation.aboveS r"
 abbreviation Above where "Above \<equiv> Order_Relation.Above r"
 abbreviation AboveS where "AboveS \<equiv> Order_Relation.AboveS r"
+abbreviation ofilter where "ofilter \<equiv> Order_Relation.ofilter r"
+lemmas ofilter_def = Order_Relation.ofilter_def[of r]
 
 
 subsection {* Auxiliaries *}
@@ -139,10 +141,6 @@
 definition suc :: "'a set \<Rightarrow> 'a"
 where "suc A \<equiv> minim (AboveS A)"
 
-definition ofilter :: "'a set \<Rightarrow> bool"
-where
-"ofilter A \<equiv> (A \<le> Field r) \<and> (\<forall>a \<in> A. under a \<le> A)"
-
 
 subsubsection {* Properties of max2 *}
 
@@ -438,7 +436,7 @@
     hence 2: "?a \<in> Field r" using minim_inField[of ?B] by blast
     have 3: "?a \<in> ?B" using minim_in[of ?B] 1 by blast
     hence 4: "?a \<notin> A" by blast
-    have 5: "A \<le> Field r" using * ofilter_def[of A] by auto
+    have 5: "A \<le> Field r" using * ofilter_def by auto
     (*  *)
     moreover
     have "A = underS ?a"