aboutsummaryrefslogtreecommitdiff
path: root/Prod.thy
diff options
context:
space:
mode:
authorJosh Chen2018-08-17 13:57:36 +0200
committerJosh Chen2018-08-17 13:57:36 +0200
commita7806604105ebf09af4237fe338c0cfcf6ebb463 (patch)
tree8cbbe1ad4d2ff668430969e21192d4d48d04a97c /Prod.thy
parenta85c05db8b3952ae07a645abfdd8b5418808cfec (diff)
Make function composition a definition instead of an axiomatization (should not need to worry about preconditions)
Diffstat (limited to 'Prod.thy')
-rw-r--r--Prod.thy10
1 files changed, 1 insertions, 9 deletions
diff --git a/Prod.thy b/Prod.thy
index 120fc59..8c94ec6 100644
--- a/Prod.thy
+++ b/Prod.thy
@@ -75,19 +75,11 @@ lemmas Prod_comps [comp] = Prod_comp Prod_uniq Prod_eq
section \<open>Function composition\<close>
-axiomatization compose :: "[Term, Term] \<Rightarrow> Term" (infixr "o" 70)
+definition compose :: "[Term, Term] \<Rightarrow> Term" (infixr "o" 70) where "g o f \<equiv> \<^bold>\<lambda>x. g`(f`x)"
syntax "_COMPOSE" :: "[Term, Term] \<Rightarrow> Term" (infixr "\<circ>" 70)
translations "g \<circ> f" \<rightleftharpoons> "g o f"
-axiomatization where
- compose_def: "\<lbrakk>
- f: A \<rightarrow> B;
- g: \<Prod>x:B. C(x);
- A \<rightarrow> B: U(i);
- (\<Prod>x:B. C(x)): U(i)
- \<rbrakk> \<Longrightarrow> g \<circ> f \<equiv> \<^bold>\<lambda>x. g`(f`x)"
-
section \<open>Unit type\<close>