| changeset 59726 | 64c2bb331035 |
| parent 58889 | 5b7a9633cfa8 |
| child 60229 | 4cd6462c1fda |
--- a/src/HOL/Lifting.thy Mon Mar 16 23:00:38 2015 +0100 +++ b/src/HOL/Lifting.thy Mon Mar 16 23:05:56 2015 +0100 @@ -376,9 +376,6 @@ lemma reflp_ge_eq: "reflp R \<Longrightarrow> R \<ge> op=" unfolding reflp_def by blast -lemma ge_eq_refl: - "R \<ge> op= \<Longrightarrow> R x x" by blast - text {* Proving a parametrized correspondence relation *} definition POS :: "('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> bool" where