aboutsummaryrefslogtreecommitdiff
path: root/Equal.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 /Equal.thy
parent8541c7d0748d06676e5eb52d61cf468858d590e2 (diff)
Library snapshot. Methods written, everything nicely organized.
Diffstat (limited to '')
-rw-r--r--Equal.thy1
1 files changed, 1 insertions, 0 deletions
diff --git a/Equal.thy b/Equal.thy
index 7732dd0..18a4207 100644
--- a/Equal.thy
+++ b/Equal.thy
@@ -9,6 +9,7 @@ theory Equal
imports HoTT_Base
begin
+
axiomatization
Equal :: "[Term, Term, Term] \<Rightarrow> Term" and
refl :: "Term \<Rightarrow> Term" ("(refl'(_'))" 1000) and