aboutsummaryrefslogtreecommitdiff
path: root/Coprod.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 /Coprod.thy
parentf83534561085c224ab30343b945ee74d1ce547f4 (diff)
Well-formation rules are back in the methods; new theory synthesizing the natural number predecessor function.
Diffstat (limited to 'Coprod.thy')
-rw-r--r--Coprod.thy14
1 files changed, 9 insertions, 5 deletions
diff --git a/Coprod.thy b/Coprod.thy
index d47c24e..178e345 100644
--- a/Coprod.thy
+++ b/Coprod.thy
@@ -44,17 +44,21 @@ and
\<And>y. y: B \<Longrightarrow> d(y): C(inr(y));
b: B
\<rbrakk> \<Longrightarrow> ind\<^sub>+(c)(d)(inr(b)) \<equiv> d(b)"
-(*
+
+
text "Admissible formation inference rules:"
axiomatization where
Coprod_form_cond1: "\<And>i A B. A + B: U(i) \<Longrightarrow> A: U(i)"
and
Coprod_form_cond2: "\<And>i A B. A + B: U(i) \<Longrightarrow> B: U(i)"
-*)
-lemmas Coprod_rules [intro] =
- Coprod_form Coprod_intro1 Coprod_intro2 Coprod_elim Coprod_comp1 Coprod_comp2
-(*lemmas Coprod_form_conds [intro] = Coprod_form_cond1 Coprod_form_cond2 *)
+
+
+text "Rule declarations:"
+
+lemmas Coprod_intro = Coprod_intro1 Coprod_intro2
+lemmas Coprod_rules [intro] = Coprod_form Coprod_intro Coprod_elim Coprod_comp1 Coprod_comp2
+lemmas Coprod_form_conds [wellform] = Coprod_form_cond1 Coprod_form_cond2
lemmas Coprod_comps [comp] = Coprod_comp1 Coprod_comp2