src/ZF/OrdQuant.thy
changeset 12667 7e6eaaa125f2
parent 12620 4e6626725e21
child 12763 6cecd9dfd53f
--- a/src/ZF/OrdQuant.thy	Tue Jan 08 15:39:47 2002 +0100
+++ b/src/ZF/OrdQuant.thy	Tue Jan 08 16:09:09 2002 +0100
@@ -36,9 +36,9 @@
   "@OUNION"   :: "[idt, i, i] => i"        ("(3\<Union>_<_./ _)" 10)
 
 
-declare Ord_Un [intro,simp]
-declare Ord_UN [intro,simp]
-declare Ord_Union [intro,simp]
+declare Ord_Un [intro,simp,TC]
+declare Ord_UN [intro,simp,TC]
+declare Ord_Union [intro,simp,TC]
 
 (** These mostly belong to theory Ordinal **)
 
@@ -49,6 +49,17 @@
 apply auto
 done
 
+lemma zero_not_Limit [iff]: "~ Limit(0)"
+by (simp add: Limit_def)
+
+lemma Limit_has_1: "Limit(i) \<Longrightarrow> 1 < i"
+by (blast intro: Limit_has_0 Limit_has_succ)
+
+lemma Limit_Union [rule_format]: "\<lbrakk>I \<noteq> 0;  \<forall>i\<in>I. Limit(i)\<rbrakk> \<Longrightarrow> Limit(\<Union>I)"
+apply (simp add: Limit_def lt_def)
+apply (blast intro!: equalityI)
+done
+
 lemma increasing_LimitI: "\<lbrakk>0<l; \<forall>x\<in>l. \<exists>y\<in>l. x<y\<rbrakk> \<Longrightarrow> Limit(l)"
 apply (simp add: Limit_def lt_Ord2)
 apply clarify