src/FOL/ex/Locale_Test/Locale_Test1.thy
changeset 67119 acb0807ddb56
parent 62020 5d208fd2507d
child 67347 bf269672c203
equal deleted inserted replaced
67118:ccab07d1196c 67119:acb0807ddb56
   724 lemma linv: "inv(x) ** x = one"
   724 lemma linv: "inv(x) ** x = one"
   725   unfolding one_def inv_def by (rule glob_linv)
   725   unfolding one_def inv_def by (rule glob_linv)
   726 
   726 
   727 end
   727 end
   728 
   728 
   729 sublocale lgrp < "def"?: dgrp
   729 sublocale lgrp < def?: dgrp
   730   rewrites one_equation: "dgrp.one(prod) = one" and inv_equation: "dgrp.inv(prod, x) = inv(x)"
   730   rewrites one_equation: "dgrp.one(prod) = one" and inv_equation: "dgrp.inv(prod, x) = inv(x)"
   731 proof -
   731 proof -
   732   show "dgrp(prod)" by unfold_locales
   732   show "dgrp(prod)" by unfold_locales
   733   from this interpret d: dgrp .
   733   from this interpret d: dgrp .
   734   \<comment> Unit
   734   \<comment> Unit