src/HOL/Lifting.thy
changeset 55083 0a689157e3ce
parent 53952 b2781a3ce958
child 55563 a64d49f49ca3
equal deleted inserted replaced
55082:e60036c1c248 55083:0a689157e3ce
   482 lemma reflp_equality: "reflp (op =)"
   482 lemma reflp_equality: "reflp (op =)"
   483 by (auto intro: reflpI)
   483 by (auto intro: reflpI)
   484 
   484 
   485 text {* Proving a parametrized correspondence relation *}
   485 text {* Proving a parametrized correspondence relation *}
   486 
   486 
   487 lemma eq_OO: "op= OO R = R"
       
   488 unfolding OO_def by metis
       
   489 
       
   490 definition POS :: "('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> bool" where
   487 definition POS :: "('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> bool" where
   491 "POS A B \<equiv> A \<le> B"
   488 "POS A B \<equiv> A \<le> B"
   492 
   489 
   493 definition  NEG :: "('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> bool" where
   490 definition  NEG :: "('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> bool" where
   494 "NEG A B \<equiv> B \<le> A"
   491 "NEG A B \<equiv> B \<le> A"