src/HOL/Transfer.thy
changeset 61630 608520e0e8e2
parent 60758 d8d85a8172b5
child 62324 ae44f16dcea5
--- a/src/HOL/Transfer.thy	Wed Nov 11 09:21:56 2015 +0100
+++ b/src/HOL/Transfer.thy	Wed Nov 11 09:48:24 2015 +0100
@@ -620,6 +620,10 @@
   shows "((A ===> B ===> op =) ===> op =) right_unique right_unique"
 unfolding right_unique_def[abs_def] by transfer_prover
 
+lemma map_fun_parametric [transfer_rule]:
+  "((A ===> B) ===> (C ===> D) ===> (B ===> C) ===> A ===> D) map_fun map_fun"
+unfolding map_fun_def[abs_def] by transfer_prover
+
 end
 
 end