aboutsummaryrefslogtreecommitdiff
path: root/Projections.thy
diff options
context:
space:
mode:
Diffstat (limited to 'Projections.thy')
-rw-r--r--Projections.thy2
1 files changed, 1 insertions, 1 deletions
diff --git a/Projections.thy b/Projections.thy
index 8ff6b30..1473e08 100644
--- a/Projections.thy
+++ b/Projections.thy
@@ -21,7 +21,7 @@ declare fst_type [intro]
lemma fst_cmp:
assumes "A: U i" and "B: A \<leadsto> U i" and "a: A" and "b: B a" shows "fst A <a, b> \<equiv> a"
-unfolding fst_def by compute (derive lems: assms)
+unfolding fst_def by (subst comp) (derive lems: assms)
declare fst_cmp [comp]