| changeset 29240 | bb81c3709fb6 | 
| parent 29237 | e90d9d51106b | 
| child 29246 | 3593802c9cf1 | 
--- a/src/HOL/Algebra/RingHom.thy Wed Dec 17 17:53:41 2008 +0100 +++ b/src/HOL/Algebra/RingHom.thy Wed Dec 17 17:53:56 2008 +0100 @@ -10,7 +10,8 @@ section {* Homomorphisms of Non-Commutative Rings *} text {* Lifting existing lemmas in a @{text ring_hom_ring} locale *} -locale ring_hom_ring = R: ring R + S: ring S + +locale ring_hom_ring = R: ring R + S: ring S + for R (structure) and S (structure) + fixes h assumes homh: "h \<in> ring_hom R S" notes hom_mult [simp] = ring_hom_mult [OF homh]