src/HOL/Transfer.thy
changeset 58128 43a1ba26a8cb
parent 57599 7ef939f89776
child 58182 82478e6c60cb
--- a/src/HOL/Transfer.thy	Mon Sep 01 16:34:39 2014 +0200
+++ b/src/HOL/Transfer.thy	Mon Sep 01 16:34:40 2014 +0200
@@ -6,7 +6,7 @@
 header {* Generic theorem transfer using relations *}
 
 theory Transfer
-imports Hilbert_Choice BNF_FP_Base Metis Option
+imports Hilbert_Choice Metis Option
 begin
 
 (* We include Option here although it's not needed here.