src/HOL/Library/FuncSet.thy
changeset 27183 0fc4c0f97a1b
parent 26106 be52145f482d
child 27368 9f90ac19e32b
equal deleted inserted replaced
27182:9e4475b9d58c 27183:0fc4c0f97a1b
   207 lemma card_bij:
   207 lemma card_bij:
   208      "[|f \<in> A\<rightarrow>B; inj_on f A;
   208      "[|f \<in> A\<rightarrow>B; inj_on f A;
   209         g \<in> B\<rightarrow>A; inj_on g B; finite A; finite B|] ==> card(A) = card(B)"
   209         g \<in> B\<rightarrow>A; inj_on g B; finite A; finite B|] ==> card(A) = card(B)"
   210   by (blast intro: card_inj order_antisym)
   210   by (blast intro: card_inj order_antisym)
   211 
   211 
   212 
       
   213 (*The following declarations generate polymorphic Skolem functions for 
       
   214   these theorems. Eventually they should become redundant, once this 
       
   215   is done automatically.*)
       
   216 
       
   217 declare FuncSet.Pi_I [skolem]
       
   218 declare FuncSet.Pi_mono [skolem]
       
   219 declare FuncSet.extensionalityI [skolem]
       
   220 declare FuncSet.funcsetI [skolem]
       
   221 declare FuncSet.restrictI [skolem]
       
   222 declare FuncSet.restrict_in_funcset [skolem]
       
   223 
       
   224 end
   212 end