src/HOL/Zorn.thy
changeset 68975 5ce4d117cea7
parent 68745 345ce5f262ea
child 69000 7cb3ddd60fd6
--- a/src/HOL/Zorn.thy	Mon Sep 10 21:33:14 2018 +0200
+++ b/src/HOL/Zorn.thy	Tue Sep 11 16:21:54 2018 +0100
@@ -376,6 +376,12 @@
   ultimately show False using * by blast
 qed
 
+lemma subset_chain_def: "\<And>\<A>. subset.chain \<A> \<C> = (\<C> \<subseteq> \<A> \<and> (\<forall>X\<in>\<C>. \<forall>Y\<in>\<C>. X \<subseteq> Y \<or> Y \<subseteq> X))"
+  by (auto simp: subset.chain_def)
+
+lemma subset_chain_insert:
+  "subset.chain \<A> (insert B \<B>) \<longleftrightarrow> B \<in> \<A> \<and> (\<forall>X\<in>\<B>. X \<subseteq> B \<or> B \<subseteq> X) \<and> subset.chain \<A> \<B>"
+  by (fastforce simp add: subset_chain_def)
 
 subsubsection \<open>Zorn's lemma\<close>