src/HOL/Equiv_Relations.thy
changeset 60517 f16e4fb20652
parent 59528 4862f3dc9540
child 60688 01488b559910
equal deleted inserted replaced
60516:0826b7025d07 60517:f16e4fb20652
   521 
   521 
   522 lemma equivp_transp:
   522 lemma equivp_transp:
   523   "equivp R \<Longrightarrow> R x y \<Longrightarrow> R y z \<Longrightarrow> R x z"
   523   "equivp R \<Longrightarrow> R x y \<Longrightarrow> R y z \<Longrightarrow> R x z"
   524   by (erule equivpE, erule transpE)
   524   by (erule equivpE, erule transpE)
   525 
   525 
       
   526 
       
   527 subsection \<open>Prominent examples\<close>
       
   528 
       
   529 lemma equivp_associated:
       
   530   "equivp associated"
       
   531 proof (rule equivpI)
       
   532   show "reflp associated"
       
   533     by (rule reflpI) simp
       
   534   show "symp associated"
       
   535     by (rule sympI) (simp add: associated_sym)
       
   536   show "transp associated"
       
   537     by (rule transpI) (fact associated_trans)
       
   538 qed
       
   539 
   526 hide_const (open) proj
   540 hide_const (open) proj
   527 
   541 
   528 end
   542 end