aboutsummaryrefslogtreecommitdiff
path: root/EqualProps.thy
diff options
context:
space:
mode:
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