src/HOL/BNF_Fixpoint_Base.thy
changeset 62335 e85c42f4f30a
parent 62325 7e4d31eefe60
child 62905 52c5a25e0c96
equal deleted inserted replaced
62334:15176172701e 62335:e85c42f4f30a
   234   by auto
   234   by auto
   235 
   235 
   236 lemma Pair_transfer: "rel_fun A (rel_fun B (rel_prod A B)) Pair Pair"
   236 lemma Pair_transfer: "rel_fun A (rel_fun B (rel_prod A B)) Pair Pair"
   237   unfolding rel_fun_def by simp
   237   unfolding rel_fun_def by simp
   238 
   238 
       
   239 lemma eq_onp_live_step: "x = y \<Longrightarrow> eq_onp P a a \<and> x \<longleftrightarrow> P a \<and> y"
       
   240   by (simp only: eq_onp_same_args)
       
   241 
       
   242 lemma top_conj: "top x \<and> P \<longleftrightarrow> P" "P \<and> top x \<longleftrightarrow> P"
       
   243   by blast+
       
   244 
   239 ML_file "Tools/BNF/bnf_fp_util.ML"
   245 ML_file "Tools/BNF/bnf_fp_util.ML"
   240 ML_file "Tools/BNF/bnf_fp_def_sugar_tactics.ML"
   246 ML_file "Tools/BNF/bnf_fp_def_sugar_tactics.ML"
   241 ML_file "Tools/BNF/bnf_fp_def_sugar.ML"
   247 ML_file "Tools/BNF/bnf_fp_def_sugar.ML"
   242 ML_file "Tools/BNF/bnf_fp_n2m_tactics.ML"
   248 ML_file "Tools/BNF/bnf_fp_n2m_tactics.ML"
   243 ML_file "Tools/BNF/bnf_fp_n2m.ML"
   249 ML_file "Tools/BNF/bnf_fp_n2m.ML"