aboutsummaryrefslogtreecommitdiff
path: root/EqualProps.thy
diff options
context:
space:
mode:
authorJosh Chen2018-09-11 19:23:21 +0200
committerJosh Chen2018-09-11 19:23:25 +0200
commitd7b9fc814d0fcb296156143a5d9bc3f5d9ad9ad1 (patch)
tree669284e48d36d8c4c1b71105077ab4bb49e19862 /EqualProps.thy
parentcd7609be19289fefe5404fce6a3fed4957ae7157 (diff)
Add the univalence axiom
Diffstat (limited to '')
-rw-r--r--EqualProps.thy2
1 files changed, 2 insertions, 0 deletions
diff --git a/EqualProps.thy b/EqualProps.thy
index 0107e8e..4cfe280 100644
--- a/EqualProps.thy
+++ b/EqualProps.thy
@@ -292,5 +292,7 @@ lemma transport_comp:
shows "transport (refl x) \<equiv> id"
unfolding transport_def by (derive lems: assms)
+text "Note that in our formulation, \<open>transport\<close> is a polymorphic function!"
+
end