aboutsummaryrefslogtreecommitdiff
path: root/Prod.thy
diff options
context:
space:
mode:
authorJosh Chen2018-07-07 23:03:33 +0200
committerJosh Chen2018-07-07 23:03:33 +0200
commitdecb363a30a30c1875bf4b93bc544c28edf3149e (patch)
treed4b8c2d5fa1b1146815c58c4630de75b6768f7c6 /Prod.thy
parent8541c7d0748d06676e5eb52d61cf468858d590e2 (diff)
Library snapshot. Methods written, everything nicely organized.
Diffstat (limited to 'Prod.thy')
-rw-r--r--Prod.thy1
1 files changed, 1 insertions, 0 deletions
diff --git a/Prod.thy b/Prod.thy
index 544a719..bf4e4e9 100644
--- a/Prod.thy
+++ b/Prod.thy
@@ -9,6 +9,7 @@ theory Prod
imports HoTT_Base
begin
+
axiomatization
Prod :: "[Term, Typefam] \<Rightarrow> Term" and
lambda :: "[Term, Term \<Rightarrow> Term] \<Rightarrow> Term" and