src/ZF/Constructible/Relative.thy
changeset 13382 b37764a46b16
parent 13363 c26eeb000470
child 13397 6e5f4d911435
--- a/src/ZF/Constructible/Relative.thy	Tue Jul 16 18:46:13 2002 +0200
+++ b/src/ZF/Constructible/Relative.thy	Tue Jul 16 18:46:59 2002 +0200
@@ -410,7 +410,7 @@
 
 text{*The class M is assumed to be transitive and to satisfy some
       relativized ZF axioms*}
-locale M_triv_axioms =
+locale (open) M_triv_axioms =
   fixes M
   assumes transM:           "[| y\<in>x; M(x) |] ==> M(y)"
       and nonempty [simp]:  "M(0)"
@@ -780,7 +780,7 @@
 
 subsection{*Some instances of separation and strong replacement*}
 
-locale M_axioms = M_triv_axioms +
+locale (open) M_axioms = M_triv_axioms +
 assumes Inter_separation:
      "M(A) ==> separation(M, \<lambda>x. \<forall>y[M]. y\<in>A --> x\<in>y)"
   and cartprod_separation: