aboutsummaryrefslogtreecommitdiff
path: root/Sum.thy
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--Sum.thy13
1 files changed, 13 insertions, 0 deletions
diff --git a/Sum.thy b/Sum.thy
index b608e75..99b4df2 100644
--- a/Sum.thy
+++ b/Sum.thy
@@ -60,4 +60,17 @@ abbreviation Pair :: "[Term, Term] \<Rightarrow> Term" (infixr "\<times>" 50)
where "A \<times> B \<equiv> \<Sum>_:A. B"
+section \<open>Null type\<close>
+
+axiomatization
+ Null :: Term ("\<zero>") and
+ indNull :: "[Typefam, Term] \<Rightarrow> Term"
+where
+ Null_form: "\<zero> : U(0)"
+and
+ Null_elim: "\<And>i C z. \<lbrakk>C: \<zero> \<longrightarrow> U(i); z : \<zero>\<rbrakk> \<Longrightarrow> indNull C z : C z"
+
+lemmas Null_rules [intro] = Null_form Null_elim
+
+
end \ No newline at end of file