src/HOL/Nominal/Nominal.thy
changeset 45625 750c5a47400b
parent 44838 096ec174be5d
child 45694 4a8743618257
equal deleted inserted replaced
45624:329bc52b4b86 45625:750c5a47400b
   376 
   376 
   377 ML {*
   377 ML {*
   378   val mksimps_pairs = (@{const_name Nominal.fresh}, @{thms fresh_prodD}) :: mksimps_pairs;
   378   val mksimps_pairs = (@{const_name Nominal.fresh}, @{thms fresh_prodD}) :: mksimps_pairs;
   379 *}
   379 *}
   380 declaration {* fn _ =>
   380 declaration {* fn _ =>
   381   Simplifier.map_ss (fn ss => ss setmksimps (mksimps mksimps_pairs))
   381   Simplifier.map_ss (Simplifier.set_mksimps (mksimps mksimps_pairs))
   382 *}
   382 *}
   383 
   383 
   384 section {* Abstract Properties for Permutations and  Atoms *}
   384 section {* Abstract Properties for Permutations and  Atoms *}
   385 (*=========================================================*)
   385 (*=========================================================*)
   386 
   386