New results from AC
authorpaulson
Thu, 06 Aug 1998 10:37:03 +0200
changeset 5262 212d203d6cd3
parent 5261 ce3c25c8a694
child 5263 8862ed2db431
New results from AC
src/ZF/Order.ML
--- a/src/ZF/Order.ML	Thu Aug 06 10:33:54 1998 +0200
+++ b/src/ZF/Order.ML	Thu Aug 06 10:37:03 1998 +0200
@@ -179,6 +179,22 @@
 qed "well_ord_0";
 
 
+(** The unit set is well-ordered by the empty relation (Grabczewski) **)
+
+Goalw [irrefl_def, trans_on_def, part_ord_def, linear_def, tot_ord_def]
+        "tot_ord({a},0)";
+by (Simp_tac 1);
+qed "tot_ord_unit";
+
+Goalw [wf_on_def, wf_def] "wf[{a}](0)";
+by (Fast_tac 1);
+qed "wf_on_unit";
+
+Goalw [well_ord_def] "well_ord({a},0)";
+by (simp_tac (simpset() addsimps [tot_ord_unit, wf_on_unit]) 1);
+qed "well_ord_unit";
+
+
 (** Order-preserving (monotone) maps **)
 
 Goalw [mono_map_def]