aboutsummaryrefslogtreecommitdiff
path: root/Sum.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 /Sum.thy
parent8541c7d0748d06676e5eb52d61cf468858d590e2 (diff)
Library snapshot. Methods written, everything nicely organized.
Diffstat (limited to '')
-rw-r--r--Sum.thy3
1 files changed, 2 insertions, 1 deletions
diff --git a/Sum.thy b/Sum.thy
index fe38960..46bb022 100644
--- a/Sum.thy
+++ b/Sum.thy
@@ -9,6 +9,7 @@ theory Sum
imports HoTT_Base
begin
+
axiomatization
Sum :: "[Term, Typefam] \<Rightarrow> Term" and
pair :: "[Term, Term] \<Rightarrow> Term" ("(1'(_,/ _'))") and
@@ -54,7 +55,7 @@ lemmas Sum_rules [intro] = Sum_form Sum_intro Sum_elim Sum_comp
lemmas Sum_form_conds [elim, wellform] = Sum_form_cond1 Sum_form_cond2
lemmas Sum_comps [comp] = Sum_comp
-\<comment> \<open>Nondependent pair\<close>
+text "Nondependent pair."
abbreviation Pair :: "[Term, Term] \<Rightarrow> Term" (infixr "\<times>" 50)
where "A \<times> B \<equiv> \<Sum>_:A. B"