aboutsummaryrefslogtreecommitdiff
path: root/Empty.thy
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--Empty.thy22
1 files changed, 9 insertions, 13 deletions
diff --git a/Empty.thy b/Empty.thy
index 107f2d7..3060867 100644
--- a/Empty.thy
+++ b/Empty.thy
@@ -1,28 +1,24 @@
-(* Title: HoTT/Empty.thy
- Author: Josh Chen
+(*
+Title: Empty.thy
+Author: Joshua Chen
+Date: 2018
Empty type
*)
theory Empty
- imports HoTT_Base
-begin
-
+imports HoTT_Base
-section \<open>Constants and type rules\<close>
+begin
-section \<open>Empty type\<close>
axiomatization
- Empty :: t ("\<zero>") and
+ Empty :: t ("\<zero>") and
indEmpty :: "t \<Rightarrow> t" ("(1ind\<^sub>\<zero>)")
where
- Empty_form: "\<zero>: U O"
-and
- Empty_elim: "\<lbrakk>C: \<zero> \<longrightarrow> U i; z: \<zero>\<rbrakk> \<Longrightarrow> ind\<^sub>\<zero> z: C z"
-
+ Empty_form: "\<zero>: U O" and
-text "Rule attribute declarations:"
+ Empty_elim: "\<lbrakk>a: \<zero>; C: \<zero> \<longrightarrow> U i\<rbrakk> \<Longrightarrow> ind\<^sub>\<zero> a: C a"
lemmas Empty_routine [intro] = Empty_form Empty_elim