--- a/src/ZF/UNITY/GenPrefix.thy Mon Feb 11 21:32:12 2008 +0100
+++ b/src/ZF/UNITY/GenPrefix.thy Mon Feb 11 21:32:13 2008 +0100
@@ -12,7 +12,7 @@
header{*Charpentier's Generalized Prefix Relation*}
theory GenPrefix
-imports Main_ZF
+imports Main
begin
definition (*really belongs in ZF/Trancl*)
--- a/src/ZF/UNITY/State.thy Mon Feb 11 21:32:12 2008 +0100
+++ b/src/ZF/UNITY/State.thy Mon Feb 11 21:32:13 2008 +0100
@@ -11,7 +11,7 @@
header{*UNITY Program States*}
-theory State imports Main_ZF begin
+theory State imports Main begin
consts var :: i
datatype var = Var("i \<in> list(nat)")