src/HOL/AxClasses/Tutorial/Group.thy
changeset 2907 0e272e4c7cb2
parent 1247 18b1441fb603
child 8920 af5e09b6c208
--- a/src/HOL/AxClasses/Tutorial/Group.thy	Fri Apr 04 16:03:11 1997 +0200
+++ b/src/HOL/AxClasses/Tutorial/Group.thy	Fri Apr 04 16:03:44 1997 +0200
@@ -19,7 +19,7 @@
 axclass
   group < semigroup
   left_unit     "1 <*> x = x"
-  left_inv      "inv x <*> x = 1"
+  left_inverse  "inverse x <*> x = 1"
 
 
 (* abelian groups *)