aboutsummaryrefslogtreecommitdiff
path: root/Proj.thy
diff options
context:
space:
mode:
authorJosh Chen2018-09-17 15:33:42 +0200
committerJosh Chen2018-09-17 15:33:42 +0200
commit8e4ca285430c7bcdabbd4ea34da38e0770f4a832 (patch)
tree1675cb6fa436e71270cb953e16895ea3071d3fe5 /Proj.thy
parent76ac8ed82317f3f62f26ecc88f412c61004bcffa (diff)
Tweak proof
Diffstat (limited to '')
-rw-r--r--Proj.thy13
1 files changed, 5 insertions, 8 deletions
diff --git a/Proj.thy b/Proj.thy
index f272224..e76e8d3 100644
--- a/Proj.thy
+++ b/Proj.thy
@@ -7,10 +7,7 @@ Projection functions \<open>fst\<close> and \<open>snd\<close> for the dependent
*)
theory Proj
-imports
- HoTT_Methods
- Prod
- Sum
+imports HoTT_Methods Prod Sum
begin
@@ -28,12 +25,12 @@ unfolding fst_def by compute (derive lems: assms)
lemma snd_type:
assumes "A: U i" and "B: A \<longrightarrow> U i" and "p: \<Sum>x:A. B x" shows "snd p: B (fst p)"
-unfolding snd_def proof
- show "\<And>p. p: \<Sum>x:A. B x \<Longrightarrow> B (fst p): U i" by (derive lems: assms fst_type)
-
+unfolding snd_def proof (derive lems: assms)
+ show "\<And>p. p: \<Sum>x:A. B x \<Longrightarrow> fst p: A" using assms(1-2) by (rule fst_type)
+
fix x y assume asm: "x: A" "y: B x"
show "y: B (fst <x,y>)" by (derive lems: asm assms fst_comp)
-qed fact
+qed
lemma snd_comp:
assumes "A: U i" and "B: A \<longrightarrow> U i" and "a: A" and "b: B a" shows "snd <a,b> \<equiv> b"