src/HOL/GroupTheory/Sylow.thy
changeset 13594 c2ee8f5a5652
parent 13583 5fcc8bf538ee
child 13595 7e6cdcd113a2
--- a/src/HOL/GroupTheory/Sylow.thy	Fri Sep 27 10:36:21 2002 +0200
+++ b/src/HOL/GroupTheory/Sylow.thy	Fri Sep 27 13:24:29 2002 +0200
@@ -71,7 +71,10 @@
 apply (simp add: calM_def, blast)
 done
 
-lemma (in sylow_central) exists_x_in_M1: "\<exists>x. x\<in>M1"
+lemma card_nonempty: "0 < card(S) ==> S \<noteq> {}"
+by force
+
+lemma (in sylow_central) exists_x_in_M1: "\<exists>x. x\<in>M1" 
 apply (subgoal_tac "0 < card M1") 
  apply (blast dest: card_nonempty) 
 apply (cut_tac prime_p [THEN prime_imp_one_less])