aboutsummaryrefslogtreecommitdiff
path: root/hott/More_Types.thy
diff options
context:
space:
mode:
authorJosh Chen2020-05-25 18:50:59 +0200
committerJosh Chen2020-05-25 18:50:59 +0200
commit60f32406e8c9712c0689d54a3dd4f8e17d310d52 (patch)
tree11fe176eb187a2f146060af1584005506f220c9d /hott/More_Types.thy
parent80edbd08e13200d2c080ac281d19948bbbcd92e0 (diff)
Lists + more reorganizing
Diffstat (limited to '')
-rw-r--r--hott/More_Types.thy (renamed from hott/Base.thy)10
1 files changed, 1 insertions, 9 deletions
diff --git a/hott/Base.thy b/hott/More_Types.thy
index 610a373..17789f8 100644
--- a/hott/Base.thy
+++ b/hott/More_Types.thy
@@ -1,17 +1,9 @@
-theory Base
+theory More_Types
imports Equivalence
begin
-section \<open>Notation\<close>
-
-syntax "_dollar" :: \<open>logic \<Rightarrow> logic \<Rightarrow> logic\<close> (infixr "$" 3)
-translations "a $ b" \<rightharpoonup> "a (b)"
-
-abbreviation (input) K where "K x \<equiv> \<lambda>_. x"
-
-
section \<open>Sum type\<close>
axiomatization