superfluous transfer rule
authorkuncar
Wed, 15 May 2013 12:10:44 +0200
changeset 51995 07344a4f19db
parent 51994 82cc2aeb7d13
child 51996 26aecb553c74
superfluous transfer rule
src/HOL/Library/FinFun.thy
--- a/src/HOL/Library/FinFun.thy	Wed May 15 12:10:39 2013 +0200
+++ b/src/HOL/Library/FinFun.thy	Wed May 15 12:10:44 2013 +0200
@@ -420,10 +420,6 @@
 lift_definition finfun_default :: "'a \<Rightarrow>f 'b \<Rightarrow> 'b"
 is "finfun_default_aux" ..
 
-lemma finfun_apply_transfer [transfer_rule]: 
-  "(fun_rel cr_finfun (fun_rel op = op =)) (\<lambda>f. f) finfun_apply"
-unfolding Rel_def fun_rel_def cr_finfun_def by simp
-
 lemma finite_finfun_default: "finite {a. finfun_apply f a \<noteq> finfun_default f}"
 by transfer (erule finite_finfun_default_aux)