aboutsummaryrefslogtreecommitdiff
path: root/Sum.thy
diff options
context:
space:
mode:
authorJosh Chen2018-07-06 10:48:41 +0200
committerJosh Chen2018-07-06 10:48:41 +0200
commit76deb7ae15fa00b5498ab43db020a0364499251e (patch)
tree706d25614154cf3767e1ad9e905a6074b620809a /Sum.thy
parentb65450369f992171f166a53e9cab408819cd987f (diff)
Added attributes to type elimination rules, not sure if these will actually be needed or useful later. Added [comp] attribute to be used by simplification met methods.
Diffstat (limited to '')
-rw-r--r--Sum.thy2
1 files changed, 2 insertions, 0 deletions
diff --git a/Sum.thy b/Sum.thy
index 1e6e6b0..93fa791 100644
--- a/Sum.thy
+++ b/Sum.thy
@@ -51,7 +51,9 @@ and
\<rbrakk> \<Longrightarrow> indSum[A,B] C f (a,b) \<equiv> f a b"
lemmas Sum_rules [intro] = Sum_form Sum_intro Sum_elim Sum_comp
+lemmas Sum_elims [dest] = Sum_elim \<comment> \<open>Declaring positively-presented dependent elimination rule as [dest] instead of [elim] arguably makes more sense.\<close>
lemmas Sum_form_conds [elim, wellform] = Sum_form_cond1 Sum_form_cond2
+lemmas Sum_comps [comp] = Sum_comp
\<comment> \<open>Nondependent pair\<close>
abbreviation Pair :: "[Term, Term] \<Rightarrow> Term" (infixr "\<times>" 50)