src/HOL/Library/Cardinality.thy
changeset 61166 5976fe402824
parent 61115 3a4400985780
child 61585 a9599d3d7610
--- a/src/HOL/Library/Cardinality.thy	Sun Sep 13 16:50:12 2015 +0200
+++ b/src/HOL/Library/Cardinality.thy	Sun Sep 13 20:20:16 2015 +0200
@@ -479,7 +479,7 @@
   and "eq_set (set ys) (List.coset xs) \<longleftrightarrow> rhs"
   and "eq_set (set xs) (set ys) \<longleftrightarrow> (\<forall>x \<in> set xs. x \<in> set ys) \<and> (\<forall>y \<in> set ys. y \<in> set xs)"
   and "eq_set (List.coset xs) (List.coset ys) \<longleftrightarrow> (\<forall>x \<in> set xs. x \<in> set ys) \<and> (\<forall>y \<in> set ys. y \<in> set xs)"
-proof goals
+proof goal_cases
   {
     case 1
     show ?case (is "?lhs \<longleftrightarrow> ?rhs")