src/HOL/Nat.thy
changeset 29652 f4c6e546b7fe
parent 29608 564ea783ace8
child 29668 33ba3faeaa0e
--- a/src/HOL/Nat.thy	Wed Jan 28 11:02:11 2009 +0100
+++ b/src/HOL/Nat.thy	Wed Jan 28 11:02:12 2009 +0100
@@ -425,6 +425,17 @@
 
 end
 
+instantiation nat :: bot
+begin
+
+definition bot_nat :: nat where
+  "bot_nat = 0"
+
+instance proof
+qed (simp add: bot_nat_def)
+
+end
+
 subsubsection {* Introduction properties *}
 
 lemma lessI [iff]: "n < Suc n"