aboutsummaryrefslogtreecommitdiff
path: root/Unit.thy
diff options
context:
space:
mode:
authorJosh Chen2019-02-22 23:45:50 +0100
committerJosh Chen2019-02-22 23:45:50 +0100
commit57d183c7955fb54b3eb6dd431f5aec338131266b (patch)
treeae6bfabbd8fcd63ee7d5140ca842599efbd58c16 /Unit.thy
parent0036345412d5c145b63693ed672b175018fa3791 (diff)
Cleanups and reorganization
Diffstat (limited to 'Unit.thy')
-rw-r--r--Unit.thy32
1 files changed, 0 insertions, 32 deletions
diff --git a/Unit.thy b/Unit.thy
deleted file mode 100644
index 7c221f0..0000000
--- a/Unit.thy
+++ /dev/null
@@ -1,32 +0,0 @@
-(*
-Title: Unit.thy
-Author: Joshua Chen
-Date: 2018
-
-Unit type
-*)
-
-theory Unit
-imports HoTT_Base
-
-begin
-
-
-axiomatization
- Unit :: t ("\<one>") and
- pt :: t ("\<star>") and
- indUnit :: "[t, t] \<Rightarrow> t" ("(1ind\<^sub>\<one>)")
-where
- Unit_form: "\<one>: U O" and
-
- Unit_intro: "\<star>: \<one>" and
-
- Unit_elim: "\<lbrakk>a: \<one>; c: C \<star>; C: \<one> \<longrightarrow> U i\<rbrakk> \<Longrightarrow> ind\<^sub>\<one> c a: C a" and
-
- Unit_comp: "\<lbrakk>c: C \<star>; C: \<one> \<longrightarrow> U i\<rbrakk> \<Longrightarrow> ind\<^sub>\<one> c \<star> \<equiv> c"
-
-lemmas Unit_form [form]
-lemmas Unit_routine [intro] = Unit_form Unit_intro Unit_elim
-lemmas Unit_comp [comp]
-
-end