From e1be5f97bb2a42b3179bc24b118d69af137f8e5d Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Sat, 18 Aug 2018 21:28:21 +0200 Subject: Regrouping type rules --- Proj.thy | 9 ++++----- 1 file changed, 4 insertions(+), 5 deletions(-) (limited to 'Proj.thy') diff --git a/Proj.thy b/Proj.thy index 291113d..dffc127 100644 --- a/Proj.thy +++ b/Proj.thy @@ -1,6 +1,5 @@ (* Title: HoTT/Proj.thy Author: Josh Chen - Date: Jun 2018 Projection functions \fst\ and \snd\ for the dependent sum type. *) @@ -27,7 +26,7 @@ lemma fst_comp: unfolding fst_def proof show "a: A" and "b: B(a)" by fact+ -qed (rule assms)+ +qed (simple lems: assms)+ lemma snd_type: assumes "\x:A. B(x): U(i)" and "p: \x:A. B(x)" shows "snd(p): B(fst p)" @@ -54,10 +53,10 @@ proof qed (simple lems: assms) -text "Rule declarations:" +text "Rule attribute declarations:" -lemmas Proj_types [intro] = fst_type snd_type -lemmas Proj_comps [comp] = fst_comp snd_comp +lemmas Proj_type [intro] = fst_type snd_type +lemmas Proj_comp [comp] = fst_comp snd_comp end -- cgit v1.2.3