aboutsummaryrefslogtreecommitdiff
path: root/Nat.thy
diff options
context:
space:
mode:
authorJosh Chen2018-08-14 17:43:03 +0200
committerJosh Chen2018-08-14 17:43:03 +0200
commite6473c383b479610cee4c0119e5811a12a938cf9 (patch)
tree477ecc678909b6e29e064ede72b9dee0933c58ad /Nat.thy
parentf83534561085c224ab30343b945ee74d1ce547f4 (diff)
Well-formation rules are back in the methods; new theory synthesizing the natural number predecessor function.
Diffstat (limited to '')
-rw-r--r--Nat.thy5
1 files changed, 5 insertions, 0 deletions
diff --git a/Nat.thy b/Nat.thy
index 388df0f..21c9b1c 100644
--- a/Nat.thy
+++ b/Nat.thy
@@ -10,6 +10,8 @@ theory Nat
begin
+section \<open>Constants and type rules\<close>
+
axiomatization
Nat :: Term ("\<nat>") and
zero :: Term ("0") and
@@ -42,6 +44,9 @@ and
n: \<nat>
\<rbrakk> \<Longrightarrow> ind\<^sub>\<nat>(f)(a)(succ n) \<equiv> f(n)(ind\<^sub>\<nat> f a n)"
+
+text "Rule declarations:"
+
lemmas Nat_intro = Nat_intro1 Nat_intro2
lemmas Nat_rules [intro] = Nat_form Nat_intro Nat_elim Nat_comp1 Nat_comp2
lemmas Nat_comps [comp] = Nat_comp1 Nat_comp2