aboutsummaryrefslogtreecommitdiff
path: root/Equal.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 /Equal.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--Equal.thy10
1 files changed, 7 insertions, 3 deletions
diff --git a/Equal.thy b/Equal.thy
index 93f623f..9fc478a 100644
--- a/Equal.thy
+++ b/Equal.thy
@@ -46,17 +46,21 @@ and
a: A
\<rbrakk> \<Longrightarrow> ind\<^sub>=(f)(refl(a)) \<equiv> f(a)"
+
text "Admissible inference rules for equality type formation:"
-(*
+
axiomatization where
Equal_form_cond1: "a =\<^sub>A b: U(i) \<Longrightarrow> A: U(i)"
and
Equal_form_cond2: "a =\<^sub>A b: U(i) \<Longrightarrow> a: A"
and
Equal_form_cond3: "a =\<^sub>A b: U(i) \<Longrightarrow> b: A"
-*)
+
+
+text "Rule declarations:"
+
lemmas Equal_rules [intro] = Equal_form Equal_intro Equal_elim Equal_comp
-(*lemmas Equal_wellform [intro] = Equal_form_cond1 Equal_form_cond2 Equal_form_cond3*)
+lemmas Equal_wellform [wellform] = Equal_form_cond1 Equal_form_cond2 Equal_form_cond3
lemmas Equal_comps [comp] = Equal_comp