src/ZF/Constructible/Reflection.thy
changeset 13382 b37764a46b16
parent 13292 f504f5d284d3
child 13428 99e52e78eb65
--- a/src/ZF/Constructible/Reflection.thy	Tue Jul 16 18:46:13 2002 +0200
+++ b/src/ZF/Constructible/Reflection.thy	Tue Jul 16 18:46:59 2002 +0200
@@ -25,7 +25,7 @@
 ultimately the @{text ex_reflection} proof is packaged up using the
 predicate @{text Reflects}.
 *}
-locale reflection =
+locale (open) reflection =
   fixes Mset and M and Reflects
   assumes Mset_mono_le : "mono_le_subset(Mset)"
       and Mset_cont    : "cont_Ord(Mset)"
@@ -124,7 +124,7 @@
 
 text{*Locale for the induction hypothesis*}
 
-locale ex_reflection = reflection +
+locale (open) ex_reflection = reflection +
   fixes P  --"the original formula"
   fixes Q  --"the reflected formula"
   fixes Cl --"the class of reflecting ordinals"
@@ -192,7 +192,7 @@
 apply (simp add: Reflects_def) 
 apply (intro conjI Closed_Unbounded_Int)
   apply blast 
- apply (rule reflection.Closed_Unbounded_ClEx [of Cl P0 Q0], blast, clarify) 
+ apply (rule Closed_Unbounded_ClEx [of Cl P0 Q0], blast, clarify) 
 apply (rule_tac Cl=Cl in  ClEx_iff, assumption+, blast) 
 done