src/HOL/Algebra/Group.thy
changeset 35416 d8d7d1b785af
parent 33057 764547b68538
child 35847 19f1f7066917
--- a/src/HOL/Algebra/Group.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/Algebra/Group.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -478,8 +478,7 @@
 
 subsection {* Direct Products *}
 
-constdefs
-  DirProd :: "_ \<Rightarrow> _ \<Rightarrow> ('a \<times> 'b) monoid"  (infixr "\<times>\<times>" 80)
+definition DirProd :: "_ \<Rightarrow> _ \<Rightarrow> ('a \<times> 'b) monoid" (infixr "\<times>\<times>" 80) where
   "G \<times>\<times> H \<equiv> \<lparr>carrier = carrier G \<times> carrier H,
                 mult = (\<lambda>(g, h) (g', h'). (g \<otimes>\<^bsub>G\<^esub> g', h \<otimes>\<^bsub>H\<^esub> h')),
                 one = (\<one>\<^bsub>G\<^esub>, \<one>\<^bsub>H\<^esub>)\<rparr>"
@@ -545,8 +544,7 @@
   "[|h \<in> hom G H; i \<in> hom H I|] ==> compose (carrier G) i h \<in> hom G I"
 by (fastsimp simp add: hom_def compose_def)
 
-constdefs
-  iso :: "_ => _ => ('a => 'b) set"  (infixr "\<cong>" 60)
+definition iso :: "_ => _ => ('a => 'b) set" (infixr "\<cong>" 60) where
   "G \<cong> H == {h. h \<in> hom G H & bij_betw h (carrier G) (carrier H)}"
 
 lemma iso_refl: "(%x. x) \<in> G \<cong> G"