src/HOL/Groups_Big.thy
changeset 63040 eb4ddd18d635
parent 62481 b5d8e57826df
child 63092 a949b2a5f51d
equal deleted inserted replaced
63039:1a20fd9cf281 63040:eb4ddd18d635
  1135     then show ?case
  1135     then show ?case
  1136     proof (cases "a = b")
  1136     proof (cases "a = b")
  1137       case True with insert show ?thesis by simp
  1137       case True with insert show ?thesis by simp
  1138     next
  1138     next
  1139       case False with insert have "a \<in> B" by simp
  1139       case False with insert have "a \<in> B" by simp
  1140       def C \<equiv> "B - {a}"
  1140       define C where "C = B - {a}"
  1141       with \<open>finite B\<close> \<open>a \<in> B\<close>
  1141       with \<open>finite B\<close> \<open>a \<in> B\<close>
  1142         have *: "B = insert a C" "finite C" "a \<notin> C" by auto
  1142         have *: "B = insert a C" "finite C" "a \<notin> C" by auto
  1143       with insert show ?thesis by (auto simp add: insert_commute ac_simps)
  1143       with insert show ?thesis by (auto simp add: insert_commute ac_simps)
  1144     qed
  1144     qed
  1145   qed
  1145   qed