aboutsummaryrefslogtreecommitdiff
path: root/HoTT_Base.thy
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--HoTT_Base.thy4
1 files changed, 2 insertions, 2 deletions
diff --git a/HoTT_Base.thy b/HoTT_Base.thy
index 34474d1..ee36af4 100644
--- a/HoTT_Base.thy
+++ b/HoTT_Base.thy
@@ -66,8 +66,8 @@ where "f: A \<leadsto> B \<equiv> (\<And>x. x: A \<Longrightarrow> f x: B)"
text \<open>We use the notation @{prop "B: A \<leadsto> U i"} to abbreviate type families.\<close>
-abbreviation (input) K_combinator :: "'a \<Rightarrow> 'b \<Rightarrow> 'a" ("^_" [1000])
-where "^A \<equiv> \<lambda>_. A"
+abbreviation (input) K_combinator :: "'a \<Rightarrow> 'b \<Rightarrow> 'a" ("&_" [0] 3)
+where "&A \<equiv> \<lambda>_. A"
section \<open>Named theorems\<close>