src/HOL/Hyperreal/NSA.thy
changeset 20485 3078fd2eec7b
parent 20432 07ec57376051
child 20541 f614c619b1e1
equal deleted inserted replaced
20484:3d3d24186352 20485:3078fd2eec7b
   545               | Const("Numeral.number_of", _) $ _ =>
   545               | Const("Numeral.number_of", _) $ _ =>
   546                                  meta_number_of_approx_reorient);
   546                                  meta_number_of_approx_reorient);
   547 
   547 
   548 in
   548 in
   549 val approx_reorient_simproc =
   549 val approx_reorient_simproc =
   550   Bin_Simprocs.prep_simproc
   550   Int_Numeral_Base_Simprocs.prep_simproc
   551     ("reorient_simproc", ["0@=x", "1@=x", "number_of w @= x"], reorient_proc);
   551     ("reorient_simproc", ["0@=x", "1@=x", "number_of w @= x"], reorient_proc);
   552 end;
   552 end;
   553 
   553 
   554 Addsimprocs [approx_reorient_simproc];
   554 Addsimprocs [approx_reorient_simproc];
   555 *}
   555 *}