src/HOL/Statespace/DistinctTreeProver.thy
changeset 32010 cb1a1c94b4cd
parent 29291 d3cc5398bad5
child 32740 9dd0a2f83429
equal deleted inserted replaced
32009:fd3c60ad9155 32010:cb1a1c94b4cd
   674                in (da := thm; thy') end)
   674                in (da := thm; thy') end)
   675 *}
   675 *}
   676 
   676 
   677 
   677 
   678 ML {* 
   678 ML {* 
   679  val ct' = cterm_of (the_context ()) t';
   679  val ct' = cterm_of @{theory} t';
   680 *}
   680 *}
   681 
   681 
   682 ML {*
   682 ML {*
   683  timeit (fn () => (DistinctTreeProver.subtractProver (term_of ct') ct' (!da);())) 
   683  timeit (fn () => (DistinctTreeProver.subtractProver (term_of ct') ct' (!da);())) 
   684 *}
   684 *}
   704 
   704 
   705 
   705 
   706 
   706 
   707 
   707 
   708 ML {*
   708 ML {*
   709 val cdist' = cterm_of (the_context ()) dist';
   709 val cdist' = cterm_of @{theory} dist';
   710 DistinctTreeProver.distinct_implProver (!da) cdist';
   710 DistinctTreeProver.distinct_implProver (!da) cdist';
   711 *}
   711 *}
   712 
   712 
   713 *)
   713 *)
   714 
   714