src/HOLCF/Pcpo.thy
changeset 22577 1a08fce38565
parent 20713 823967ef47f1
child 25131 2c8caac48ade
equal deleted inserted replaced
22576:1beba4e2aa9f 22577:1a08fce38565
   204       | Const("HOL.one", _) => NONE
   204       | Const("HOL.one", _) => NONE
   205       | Const("Numeral.number_of", _) $ _ => NONE
   205       | Const("Numeral.number_of", _) $ _ => NONE
   206       | _ => SOME meta_UU_reorient;
   206       | _ => SOME meta_UU_reorient;
   207 in
   207 in
   208   val UU_reorient_simproc = 
   208   val UU_reorient_simproc = 
   209     Simplifier.simproc (the_context ())
   209     Simplifier.simproc @{theory} "UU_reorient_simproc" ["UU=x"] reorient_proc
   210       "UU_reorient_simproc" ["UU=x"] reorient_proc
       
   211 end;
   210 end;
   212 
   211 
   213 Addsimprocs [UU_reorient_simproc];
   212 Addsimprocs [UU_reorient_simproc];
   214 *}
   213 *}
   215 
   214