src/HOL/Code_Evaluation.thy
changeset 52143 36ffe23b25f8
parent 51160 599ff65b85e2
child 52286 8170e5327c02
equal deleted inserted replaced
52142:348aed032cda 52143:36ffe23b25f8
   142 
   142 
   143 
   143 
   144 subsubsection {* Obfuscation *}
   144 subsubsection {* Obfuscation *}
   145 
   145 
   146 print_translation {*
   146 print_translation {*
   147 let
   147   let
   148   val term = Const ("<TERM>", dummyT);
   148     val term = Const ("<TERM>", dummyT);
   149   fun tr1' [_, _] = term;
   149     fun tr1' _ [_, _] = term;
   150   fun tr2' [] = term;
   150     fun tr2' _ [] = term;
   151 in
   151   in
   152   [(@{const_syntax Const}, tr1'),
   152    [(@{const_syntax Const}, tr1'),
   153     (@{const_syntax App}, tr1'),
   153     (@{const_syntax App}, tr1'),
   154     (@{const_syntax dummy_term}, tr2')]
   154     (@{const_syntax dummy_term}, tr2')]
   155 end
   155   end
   156 *}
   156 *}
   157 
   157 
   158 
   158 
   159 subsection {* Diagnostic *}
   159 subsection {* Diagnostic *}
   160 
   160