| changeset 69700 | 7a92cbec7030 |
| parent 69593 | 3dda49e08b9d |
| child 70019 | 095dce9892e8 |
--- a/src/HOL/Real_Vector_Spaces.thy Sun Jan 20 17:15:49 2019 +0000 +++ b/src/HOL/Real_Vector_Spaces.thy Mon Jan 21 14:44:23 2019 +0000 @@ -322,7 +322,7 @@ instance real_algebra_1 < ring_char_0 proof from inj_of_real inj_of_nat have "inj (of_real \<circ> of_nat)" - by (rule inj_comp) + by (rule inj_compose) then show "inj (of_nat :: nat \<Rightarrow> 'a)" by (simp add: comp_def) qed