src/HOL/Relation.thy
changeset 76574 7bc934b99faf
parent 76573 cbf38b7cb195
child 76588 82a36e3d1b55
equal deleted inserted replaced
76573:cbf38b7cb195 76574:7bc934b99faf
   559   by (blast intro: transI)
   559   by (blast intro: transI)
   560 
   560 
   561 lemma transp_singleton [simp]: "transp (\<lambda>x y. x = a \<and> y = a)"
   561 lemma transp_singleton [simp]: "transp (\<lambda>x y. x = a \<and> y = a)"
   562   by (simp add: transp_def)
   562   by (simp add: transp_def)
   563 
   563 
       
   564 lemma asym_if_irrefl_and_trans: "irrefl R \<Longrightarrow> trans R \<Longrightarrow> asym R"
       
   565   by (auto intro: asymI dest: transD irreflD)
       
   566 
       
   567 lemma asymp_if_irreflp_and_transp: "irreflp R \<Longrightarrow> transp R \<Longrightarrow> asymp R"
       
   568   by (rule asym_if_irrefl_and_trans[to_pred])
       
   569 
   564 context preorder
   570 context preorder
   565 begin
   571 begin
   566 
   572 
   567 lemma transp_le[simp]: "transp (\<le>)"
   573 lemma transp_le[simp]: "transp (\<le>)"
   568 by(auto simp add: transp_def intro: order_trans)
   574 by(auto simp add: transp_def intro: order_trans)