Datasets:

Modalities:
Text
Languages:
English
Libraries:
Datasets
License:
proof-pile / formal /afp /Automatic_Refinement /Automatic_Refinement.thy
Zhangir Azerbayev
squashed?
4365a98
raw
history blame
1.16 kB
section \<open>Entry Point for the Automatic Refinement Tool\<close>
theory Automatic_Refinement
imports
"Tool/Autoref_Tool"
Autoref_Bindings_HOL
begin
text \<open>The automatic refinement tool should be used by
importing this theory\<close>
subsection \<open>Convenience\<close>
text \<open>The following lemmas can be used to add tags to theorems\<close>
lemma PREFER_I: "P x \<Longrightarrow> PREFER P x" by simp
lemma PREFER_D: "PREFER P x \<Longrightarrow> P x" by simp
lemmas PREFER_sv_D = PREFER_D[of single_valued]
lemma PREFER_id_D: "PREFER_id R \<Longrightarrow> R=Id" by simp
abbreviation "PREFER_RUNIV \<equiv> PREFER (\<lambda>R. Range R = UNIV)"
lemmas PREFER_RUNIV_D = PREFER_D[of "(\<lambda>R. Range R = UNIV)"]
lemma SIDE_GEN_ALGO_D: "SIDE_GEN_ALGO P \<Longrightarrow> P" by simp
lemma GEN_OP_D: "GEN_OP c a R \<Longrightarrow> (c,a)\<in>R"
by simp
lemma MINOR_PRIO_TAG_I: "P \<Longrightarrow> (MINOR_PRIO_TAG p \<Longrightarrow> P)" by auto
lemma MAJOR_PRIO_TAG_I: "P \<Longrightarrow> (MAJOR_PRIO_TAG p \<Longrightarrow> P)" by auto
lemma PRIO_TAG_I: "P \<Longrightarrow> (PRIO_TAG ma mi \<Longrightarrow> P)" by auto
end