src/HOL/Decision_Procs/Dense_Linear_Order.thy
changeset 69605 a96320074298
parent 69597 ff784d5a5bfb
child 74397 e80c4cde6064
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
     7 
     7 
     8 theory Dense_Linear_Order
     8 theory Dense_Linear_Order
     9 imports Main
     9 imports Main
    10 begin
    10 begin
    11 
    11 
    12 ML_file "langford_data.ML"
    12 ML_file \<open>langford_data.ML\<close>
    13 ML_file "ferrante_rackoff_data.ML"
    13 ML_file \<open>ferrante_rackoff_data.ML\<close>
    14 
    14 
    15 context linorder
    15 context linorder
    16 begin
    16 begin
    17 
    17 
    18 lemma less_not_permute[no_atp]: "\<not> (x < y \<and> y < x)"
    18 lemma less_not_permute[no_atp]: "\<not> (x < y \<and> y < x)"
   422 lemma ex_distrib[no_atp]: "(\<exists>x. P x \<or> Q x) \<longleftrightarrow> ((\<exists>x. P x) \<or> (\<exists>x. Q x))"
   422 lemma ex_distrib[no_atp]: "(\<exists>x. P x \<or> Q x) \<longleftrightarrow> ((\<exists>x. P x) \<or> (\<exists>x. Q x))"
   423   by blast
   423   by blast
   424 
   424 
   425 lemmas dnf_simps[no_atp] = weak_dnf_simps nnf_simps ex_distrib
   425 lemmas dnf_simps[no_atp] = weak_dnf_simps nnf_simps ex_distrib
   426 
   426 
   427 ML_file "langford.ML"
   427 ML_file \<open>langford.ML\<close>
   428 method_setup dlo = \<open>
   428 method_setup dlo = \<open>
   429   Scan.succeed (SIMPLE_METHOD' o Langford.dlo_tac)
   429   Scan.succeed (SIMPLE_METHOD' o Langford.dlo_tac)
   430 \<close> "Langford's algorithm for quantifier elimination in dense linear orders"
   430 \<close> "Langford's algorithm for quantifier elimination in dense linear orders"
   431 
   431 
   432 
   432 
   744 end
   744 end
   745 \<close>
   745 \<close>
   746 
   746 
   747 end
   747 end
   748 
   748 
   749 ML_file "ferrante_rackoff.ML"
   749 ML_file \<open>ferrante_rackoff.ML\<close>
   750 
   750 
   751 method_setup ferrack = \<open>
   751 method_setup ferrack = \<open>
   752   Scan.succeed (SIMPLE_METHOD' o FerranteRackoff.dlo_tac)
   752   Scan.succeed (SIMPLE_METHOD' o FerranteRackoff.dlo_tac)
   753 \<close> "Ferrante and Rackoff's algorithm for quantifier elimination in dense linear orders"
   753 \<close> "Ferrante and Rackoff's algorithm for quantifier elimination in dense linear orders"
   754 
   754