src/HOL/Dense_Linear_Order.thy
changeset 23466 886655a150f6
parent 23453 bf46f5cbdd64
child 23470 e28b41e8b7d4
equal deleted inserted replaced
23465:8f8835aac299 23466:886655a150f6
     7   and a quantifier elimination procedure in Ferrante and Rackoff style *}
     7   and a quantifier elimination procedure in Ferrante and Rackoff style *}
     8 
     8 
     9 theory Dense_Linear_Order
     9 theory Dense_Linear_Order
    10 imports Finite_Set
    10 imports Finite_Set
    11 uses
    11 uses
    12   "Tools/qelim.ML"
    12   "Tools/Qelim/qelim.ML"
    13   "Tools/Ferrante_Rackoff/ferrante_rackoff_data.ML"
    13   "Tools/Qelim/ferrante_rackoff_data.ML"
    14   ("Tools/Ferrante_Rackoff/ferrante_rackoff.ML")
    14   ("Tools/Qelim/ferrante_rackoff.ML")
    15 begin
    15 begin
    16 
    16 
    17 setup Ferrante_Rackoff_Data.setup
    17 setup Ferrante_Rackoff_Data.setup
    18 
    18 
    19 context Linorder
    19 context Linorder
   413 end
   413 end
   414 *}
   414 *}
   415 
   415 
   416 end
   416 end
   417 
   417 
   418 use "Tools/Ferrante_Rackoff/ferrante_rackoff.ML"
   418 use "Tools/Qelim/ferrante_rackoff.ML"
   419 
   419 
   420 method_setup dlo = {*
   420 method_setup dlo = {*
   421   Method.ctxt_args (Method.SIMPLE_METHOD' o FerranteRackoff.dlo_tac)
   421   Method.ctxt_args (Method.SIMPLE_METHOD' o FerranteRackoff.dlo_tac)
   422 *} "Ferrante and Rackoff's algorithm for quantifier elimination in dense linear orders"
   422 *} "Ferrante and Rackoff's algorithm for quantifier elimination in dense linear orders"
   423 
   423