src/Doc/Classes/Classes.thy
changeset 62939 ef8d840f39fb
parent 61566 c3d6e570ccef
child 67406 23307fd33906
--- a/src/Doc/Classes/Classes.thy	Sat Apr 09 20:38:08 2016 +0200
+++ b/src/Doc/Classes/Classes.thy	Sat Apr 09 21:42:42 2016 +0200
@@ -146,7 +146,7 @@
   @{command definition}).  The concluding @{command instance} opens a
   proof that the given parameters actually conform to the class
   specification.  Note that the first proof step is the @{method
-  default} method, which for such instance proofs maps to the @{method
+  standard} method, which for such instance proofs maps to the @{method
   intro_classes} method.  This reduces an instance judgement to the
   relevant primitive proof goals; typically it is the first method
   applied in an instantiation proof.