changeset 349 | f507f088de73 |
parent 348 | b1f83c7a8674 |
child 351 | 3aba0cf85f97 |
--- a/QuotMain.thy Mon Nov 23 21:12:16 2009 +0100 +++ b/QuotMain.thy Mon Nov 23 21:48:44 2009 +0100 @@ -1264,7 +1264,7 @@ in if ty = ty' then Const (@{const_name "op ="}, ty) $ subtrm - else mk_resp_arg lthy (ty, ty') $ subtrm + else mk_resp_arg lthy (domain_type ty, domain_type ty') $ subtrm end | (t1 $ t2, t1' $ t2') => (REGULARIZE_trm lthy t1 t1') $ (REGULARIZE_trm lthy t2 t2')