imports Main;
authorwenzelm
Mon, 11 Feb 2008 21:32:13 +0100
changeset 26060 cd89870aa92f
parent 26059 b67a225b50fd
child 26061 59de52bec3ec
imports Main;
src/ZF/UNITY/GenPrefix.thy
src/ZF/UNITY/State.thy
--- 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)")