Nominal-General/Nominal2_Eqvt.thy
changeset 1866 6d4e4bf9bce6
parent 1835 636de31888a6
child 1867 f4477d3fe520
equal deleted inserted replaced
1865:b71b838b0a75 1866:6d4e4bf9bce6
   367 
   367 
   368 declare [[trace_eqvt = false]]
   368 declare [[trace_eqvt = false]]
   369 
   369 
   370 text {* Problem: there is no raw eqvt-rule for The *}
   370 text {* Problem: there is no raw eqvt-rule for The *}
   371 lemma "p \<bullet> (THE x. P x) = foo"
   371 lemma "p \<bullet> (THE x. P x) = foo"
       
   372 apply(tactic {* Nominal_Permeq.eqvt_tac @{context} [] [@{const_name "The"}] 1*})
   372 apply(perm_simp)
   373 apply(perm_simp)
   373 (* apply(perm_strict_simp) *)
   374 (* apply(perm_strict_simp) *)
   374 oops
   375 oops
   375 
   376 
   376 (* automatic equivariance procedure for 
   377 (* automatic equivariance procedure for