src/ZF/Coind/Static.thy
changeset 76214 0c18df79b1c8
parent 76213 e44d86131648
child 76215 a642599ffdea
--- a/src/ZF/Coind/Static.thy	Tue Sep 27 16:51:35 2022 +0100
+++ b/src/ZF/Coind/Static.thy	Tue Sep 27 17:03:23 2022 +0100
@@ -17,9 +17,9 @@
 definition
   isofenv :: "[i,i] => o"  where
    "isofenv(ve,te) \<equiv>                
-      ve_dom(ve) = te_dom(te) &            
+      ve_dom(ve) = te_dom(te) \<and>            
       (\<forall>x \<in> ve_dom(ve).                          
-        \<exists>c \<in> Const. ve_app(ve,x) = v_const(c) & isof(c,te_app(te,x)))"
+        \<exists>c \<in> Const. ve_app(ve,x) = v_const(c) \<and> isof(c,te_app(te,x)))"
   
 
 (*** Elaboration ***)