src/HOL/Multivariate_Analysis/Finite_Cartesian_Product.thy
changeset 33715 8cce3a34c122
parent 33175 2083bde13ce1
child 34289 c9c14c72d035
--- a/src/HOL/Multivariate_Analysis/Finite_Cartesian_Product.thy	Mon Nov 16 15:06:34 2009 +0100
+++ b/src/HOL/Multivariate_Analysis/Finite_Cartesian_Product.thy	Mon Nov 16 15:03:23 2009 +0100
@@ -8,15 +8,6 @@
 imports Main (*FIXME: ATP_Linkup is only needed for metis at a few places. We could dispense of that by changing the proofs.*)
 begin
 
-definition hassize (infixr "hassize" 12) where
-  "(S hassize n) = (finite S \<and> card S = n)"
-
-lemma hassize_image_inj: assumes f: "inj_on f S" and S: "S hassize n"
-  shows "f ` S hassize n"
-  using f S card_image[OF f]
-    by (simp add: hassize_def inj_on_def)
-
-
 subsection {* Finite Cartesian products, with indexing and lambdas. *}
 
 typedef (open Cart)