| changeset 22274 | ce1459004c8d |
| parent 21404 | eb85850d3eb7 |
| child 23755 | 1c4672d130b1 |
--- a/src/HOL/NumberTheory/BijectionRel.thy Wed Feb 07 17:46:03 2007 +0100 +++ b/src/HOL/NumberTheory/BijectionRel.thy Wed Feb 07 17:51:38 2007 +0100 @@ -71,7 +71,7 @@ "!!F a. F \<subseteq> A ==> a \<in> A ==> a \<notin> F ==> P F ==> P (insert a F)" shows "P F" using major subs - apply (induct set: Finites) + apply (induct set: finite) apply (blast intro: cases)+ done