src/HOL/BNF_Def.thy
changeset 63714 b62f4f765353
parent 63092 a949b2a5f51d
child 63834 6a757f36997e
--- a/src/HOL/BNF_Def.thy	Wed Aug 17 16:16:38 2016 +0200
+++ b/src/HOL/BNF_Def.thy	Thu Aug 18 11:10:07 2016 +0200
@@ -269,6 +269,9 @@
   "rel_fun A B f g \<Longrightarrow> X \<subseteq> Collect (case_prod A) \<Longrightarrow> x \<in> X \<Longrightarrow> B ((f o fst) x) ((g o snd) x)"
   unfolding rel_fun_def by auto
 
+lemma eq_onp_mono_iff: "eq_onp P \<le> eq_onp Q \<longleftrightarrow> P \<le> Q"
+  unfolding eq_onp_def by auto
+
 ML_file "Tools/BNF/bnf_util.ML"
 ML_file "Tools/BNF/bnf_tactics.ML"
 ML_file "Tools/BNF/bnf_def_tactics.ML"