# HG changeset patch # User Andreas Lochbihler # Date 1469789062 -7200 # Node ID 0bcd79da075b0e2ffe65a1a47fee095cedc6ff62 # Parent 6f7a9d48a82879db8a431eea450132d02da6081d prefer [simp] over [iff] as [iff] break HOL-UNITY diff -r 6f7a9d48a828 -r 0bcd79da075b src/HOL/Order_Relation.thy --- a/src/HOL/Order_Relation.thy Fri Jul 29 11:42:13 2016 +0200 +++ b/src/HOL/Order_Relation.thy Fri Jul 29 12:44:22 2016 +0200 @@ -55,7 +55,7 @@ "linear_order_on A r \ strict_linear_order_on A (r-Id)" by(simp add: order_on_defs trans_diff_Id) -lemma linear_order_on_singleton [iff]: "linear_order_on {x} {(x, x)}" +lemma linear_order_on_singleton [simp]: "linear_order_on {x} {(x, x)}" unfolding order_on_defs by simp lemma linear_order_on_acyclic: diff -r 6f7a9d48a828 -r 0bcd79da075b src/HOL/Relation.thy --- a/src/HOL/Relation.thy Fri Jul 29 11:42:13 2016 +0200 +++ b/src/HOL/Relation.thy Fri Jul 29 12:44:22 2016 +0200 @@ -206,7 +206,7 @@ lemma refl_on_empty [simp]: "refl_on {} {}" by (simp add: refl_on_def) -lemma refl_on_singleton [iff]: "refl_on {x} {(x, x)}" +lemma refl_on_singleton [simp]: "refl_on {x} {(x, x)}" by (blast intro: refl_onI) lemma refl_on_def' [nitpick_unfold, code]: @@ -338,7 +338,7 @@ lemma antisymP_equality [simp]: "antisymP op =" by (auto intro: antisymI) -lemma antisym_singleton [iff]: "antisym {x}" +lemma antisym_singleton [simp]: "antisym {x}" by (blast intro: antisymI) @@ -399,16 +399,16 @@ lemma transp_equality [simp]: "transp op =" by (auto intro: transpI) -lemma trans_empty [iff]: "trans {}" +lemma trans_empty [simp]: "trans {}" by (blast intro: transI) -lemma transp_empty [iff]: "transp (\x y. False)" +lemma transp_empty [simp]: "transp (\x y. False)" using trans_empty[to_pred] by(simp add: bot_fun_def) -lemma trans_singleton [iff]: "trans {(a, a)}" +lemma trans_singleton [simp]: "trans {(a, a)}" by (blast intro: transI) -lemma transp_singleton [iff]: "transp (\x y. x = a \ y = a)" +lemma transp_singleton [simp]: "transp (\x y. x = a \ y = a)" by(simp add: transp_def) subsubsection \Totality\ @@ -425,7 +425,7 @@ lemma total_on_empty [simp]: "total_on {} r" by (simp add: total_on_def) -lemma total_on_singleton [iff]: "total_on {x} {(x, x)}" +lemma total_on_singleton [simp]: "total_on {x} {(x, x)}" unfolding total_on_def by blast subsubsection \Single valued relations\ @@ -931,7 +931,7 @@ lemma Domain_unfold: "Domain r = {x. \y. (x, y) \ r}" by blast -lemma Field_square [iff]: "Field (x \ x) = x" +lemma Field_square [simp]: "Field (x \ x) = x" unfolding Field_def by blast