src/HOL/Nat.thy
changeset 58306 117ba6cbe414
parent 58189 9d714be4f028
child 58377 c6f93b8d2d8e
--- a/src/HOL/Nat.thy	Thu Sep 11 18:54:36 2014 +0200
+++ b/src/HOL/Nat.thy	Thu Sep 11 18:54:36 2014 +0200
@@ -96,10 +96,10 @@
   apply (simp only: Suc_not_Zero)
   done
 
--- {* Avoid name clashes by prefixing the output of @{text rep_datatype} with @{text old}. *}
+-- {* Avoid name clashes by prefixing the output of @{text old_rep_datatype} with @{text old}. *}
 setup {* Sign.mandatory_path "old" *}
 
-rep_datatype "0 \<Colon> nat" Suc
+old_rep_datatype "0 \<Colon> nat" Suc
   apply (erule nat_induct0, assumption)
  apply (rule nat.inject)
 apply (rule nat.distinct(1))