aboutsummaryrefslogtreecommitdiff
path: root/mltt/lib/List.thy
diff options
context:
space:
mode:
authorJosh Chen2021-06-24 22:40:05 +0100
committerJosh Chen2021-06-24 22:40:05 +0100
commitf988d541364841cd208f4fd21ff8e5e2935fc7aa (patch)
tree8ccc4d4e4cdde7572453ac0e250a224fe8db3da1 /mltt/lib/List.thy
parent0085798a86a35e2430a97289e894724f688db435 (diff)
Bad practice huge commit:
1. Rudimentary prototype definitional package 2. Started univalence 3. Various compatibility fixes and new theory stubs 4. Updated ROOT file
Diffstat (limited to 'mltt/lib/List.thy')
-rw-r--r--mltt/lib/List.thy10
1 files changed, 5 insertions, 5 deletions
diff --git a/mltt/lib/List.thy b/mltt/lib/List.thy
index 4beb9b6..0cd43c8 100644
--- a/mltt/lib/List.thy
+++ b/mltt/lib/List.thy
@@ -83,7 +83,7 @@ section \<open>Standard functions\<close>
subsection \<open>Head and tail\<close>
-Definition head:
+Lemma (def) head:
assumes "A: U i" "xs: List A"
shows "Maybe A"
proof (cases xs)
@@ -91,7 +91,7 @@ proof (cases xs)
show "\<And>x. x: A \<Longrightarrow> some x: Maybe A" by intro
qed
-Definition tail:
+Lemma (def) tail:
assumes "A: U i" "xs: List A"
shows "List A"
proof (cases xs)
@@ -128,7 +128,7 @@ Lemma tail_of_cons [comp]:
subsection \<open>Append\<close>
-Definition app:
+Lemma (def) app:
assumes "A: U i" "xs: List A" "ys: List A"
shows "List A"
apply (elim xs)
@@ -143,7 +143,7 @@ translations "app" \<leftharpoondown> "CONST List.app A"
subsection \<open>Map\<close>
-Definition map:
+Lemma (def) map:
assumes "A: U i" "B: U i" "f: A \<rightarrow> B" "xs: List A"
shows "List B"
proof (elim xs)
@@ -165,7 +165,7 @@ Lemma map_type [type]:
subsection \<open>Reverse\<close>
-Definition rev:
+Lemma (def) rev:
assumes "A: U i" "xs: List A"
shows "List A"
apply (elim xs)