src/HOL/Library/Eval.thy
changeset 26032 377b7aa0b5b5
parent 26020 ffe1a032d24b
child 26037 8bf9e480a7b8
equal deleted inserted replaced
26031:9830e7ffd574 26032:377b7aa0b5b5
   306     -- OuterParse.term
   306     -- OuterParse.term
   307       >> (fn (some_name, t) => Toplevel.no_timing o Toplevel.keep
   307       >> (fn (some_name, t) => Toplevel.no_timing o Toplevel.keep
   308            (Eval.evaluate_cmd some_name t)));
   308            (Eval.evaluate_cmd some_name t)));
   309 *}
   309 *}
   310 
   310 
   311 hide (open) const Type TFree Const App dummy_term typ_of term_of
   311 print_translation {*
   312 
   312 let
   313 end
   313   val term = Const ("<TERM>", dummyT);
       
   314   fun tr1' [_, _] = term;
       
   315   fun tr2' [] = term;
       
   316 in
       
   317   [(@{const_syntax Const}, tr1'),
       
   318     (@{const_syntax App}, tr1'),
       
   319     (@{const_syntax dummy_term}, tr2')]
       
   320 end
       
   321 *}
       
   322 
       
   323 hide (open) const Type TFree typ_of term_of
       
   324 hide const Const App dummy_term
       
   325 
       
   326 end