src/HOL/BNF/Basic_BNFs.thy
changeset 52545 d2ad6eae514f
parent 51893 596baae88a88
child 52635 4f84b730c489
--- a/src/HOL/BNF/Basic_BNFs.thy	Fri Jul 05 18:10:07 2013 +0200
+++ b/src/HOL/BNF/Basic_BNFs.thy	Sun Jul 07 10:24:00 2013 +0200
@@ -317,7 +317,7 @@
 lemma card_of_bounded_range:
   "|{f :: 'd \<Rightarrow> 'a. range f \<subseteq> B}| \<le>o |Func (UNIV :: 'd set) B|" (is "|?LHS| \<le>o |?RHS|")
 proof -
-  let ?f = "\<lambda>f. %x. if f x \<in> B then Some (f x) else None"
+  let ?f = "\<lambda>f. %x. if f x \<in> B then f x else undefined"
   have "inj_on ?f ?LHS" unfolding inj_on_def
   proof (unfold fun_eq_iff, safe)
     fix g :: "'d \<Rightarrow> 'a" and f :: "'d \<Rightarrow> 'a" and x