src/HOL/Groups_List.thy
changeset 64272 f76b6dda2e56
parent 64267 b9a1486e79be
child 66308 b6a0d95b94be
--- a/src/HOL/Groups_List.thy	Mon Oct 17 14:37:32 2016 +0200
+++ b/src/HOL/Groups_List.thy	Mon Oct 17 17:33:07 2016 +0200
@@ -340,15 +340,15 @@
   from prod_list_def show "monoid_list.F times 1 = prod_list" by simp
 qed
 
-sublocale setprod: comm_monoid_list_set times 1
+sublocale prod: comm_monoid_list_set times 1
 rewrites
   "monoid_list.F times 1 = prod_list"
-  and "comm_monoid_set.F times 1 = setprod"
+  and "comm_monoid_set.F times 1 = prod"
 proof -
   show "comm_monoid_list_set times 1" ..
-  then interpret setprod: comm_monoid_list_set times 1 .
+  then interpret prod: comm_monoid_list_set times 1 .
   from prod_list_def show "monoid_list.F times 1 = prod_list" by simp
-  from setprod_def show "comm_monoid_set.F times 1 = setprod" by (auto intro: sym)
+  from prod_def show "comm_monoid_set.F times 1 = prod" by (auto intro: sym)
 qed
 
 end