src/HOL/BNF_Examples/TreeFsetI.thy
changeset 55129 26bd1cba3ab5
parent 55091 c43394c2e5ec
child 55933 12ee2c407dad
--- a/src/HOL/BNF_Examples/TreeFsetI.thy	Thu Jan 23 19:02:22 2014 +0100
+++ b/src/HOL/BNF_Examples/TreeFsetI.thy	Fri Jan 24 11:51:45 2014 +0100
@@ -9,7 +9,7 @@
 header {* Finitely Branching Possibly Infinite Trees, with Sets of Children *}
 
 theory TreeFsetI
-imports "~~/src/HOL/Library/More_BNFs"
+imports "~~/src/HOL/Library/FSet"
 begin
 
 codatatype 'a treeFsetI = Tree (lab: 'a) (sub: "'a treeFsetI fset")