# HG changeset patch # User wenzelm # Date 1632080830 -7200 # Node ID dd04da556d1a57725821fce37d8360422b0f9f31 # Parent 54b2e5f771daf27f1c23c3986b60cd8347e8add6 clarified antiquotations; diff -r 54b2e5f771da -r dd04da556d1a src/FOL/fologic.ML --- a/src/FOL/fologic.ML Sun Sep 19 21:37:14 2021 +0200 +++ b/src/FOL/fologic.ML Sun Sep 19 21:47:10 2021 +0200 @@ -15,16 +15,12 @@ val dest_conj: term -> term list val mk_iff: term * term -> term val dest_iff: term -> term * term - val all_const: typ -> term val mk_all: term * term -> term - val exists_const: typ -> term val mk_exists: term * term -> term - val eq_const: typ -> term val mk_eq: term * term -> term val dest_eq: term -> term * term end; - structure FOLogic: FOLOGIC = struct @@ -44,15 +40,13 @@ val dest_iff = \<^Const_fn>\iff for A B => \(A, B)\\; -fun eq_const T = \<^Const>\eq T\; -fun mk_eq (t, u) = eq_const (fastype_of t) $ t $ u; +fun mk_eq (t, u) = + let val T = fastype_of t + in \<^Const>\eq T for t u\ end; val dest_eq = \<^Const_fn>\eq _ for lhs rhs => \(lhs, rhs)\\; -fun all_const T = \<^Const>\All T\; -fun mk_all (Free (x, T), P) = all_const T $ absfree (x, T) P; - -fun exists_const T = \<^Const>\Ex T\; -fun mk_exists (Free (x, T), P) = exists_const T $ absfree (x, T) P; +fun mk_all (Free (x, T), P) = \<^Const>\All T for \absfree (x, T) P\\; +fun mk_exists (Free (x, T), P) = \<^Const>\Ex T for \absfree (x, T) P\\; end; diff -r 54b2e5f771da -r dd04da556d1a src/ZF/ind_syntax.ML --- a/src/ZF/ind_syntax.ML Sun Sep 19 21:37:14 2021 +0200 +++ b/src/ZF/ind_syntax.ML Sun Sep 19 21:47:10 2021 +0200 @@ -20,8 +20,10 @@ (*Creates All(%v.v:A --> P(v)) rather than Ball(A,P) *) fun mk_all_imp (A,P) = - FOLogic.all_const \<^Type>\i\ $ - Abs("v", \<^Type>\i\, \<^Const>\imp\ $ \<^Const>\mem for \Bound 0\ A\ $ Term.betapply(P, Bound 0)); + let val T = \<^Type>\i\ in + \<^Const>\All T for + \Abs ("v", T, \<^Const>\imp for \\<^Const>\mem for \Bound 0\ A\\ \Term.betapply (P, Bound 0)\\)\\ + end; fun mk_Collect (a, D, t) = \<^Const>\Collect for D\ $ absfree (a, \<^Type>\i\) t;