src/ZF/Constructible/L_axioms.thy
changeset 13385 31df66ca0780
parent 13363 c26eeb000470
child 13418 7c0ba9dba978
equal deleted inserted replaced
13384:a34e38154413 13385:31df66ca0780
   370                \<lambda>i x. empty(**Lset(i),f(x))]"
   370                \<lambda>i x. empty(**Lset(i),f(x))]"
   371 apply (simp only: empty_def setclass_simps)
   371 apply (simp only: empty_def setclass_simps)
   372 apply (intro FOL_reflections)  
   372 apply (intro FOL_reflections)  
   373 done
   373 done
   374 
   374 
       
   375 text{*Not used.  But maybe useful?*}
       
   376 lemma Transset_sats_empty_fm_eq_0:
       
   377    "[| n \<in> nat; env \<in> list(A); Transset(A)|]
       
   378     ==> sats(A, empty_fm(n), env) <-> nth(n,env) = 0"
       
   379 apply (simp add: empty_fm_def empty_def Transset_def, auto)
       
   380 apply (case_tac "n < length(env)") 
       
   381 apply (frule nth_type, assumption+, blast)  
       
   382 apply (simp_all add: not_lt_iff_le nth_eq_0) 
       
   383 done
       
   384 
   375 
   385 
   376 subsubsection{*Unordered Pairs, Internalized*}
   386 subsubsection{*Unordered Pairs, Internalized*}
   377 
   387 
   378 constdefs upair_fm :: "[i,i,i]=>i"
   388 constdefs upair_fm :: "[i,i,i]=>i"
   379     "upair_fm(x,y,z) == 
   389     "upair_fm(x,y,z) ==