src/ZF/ind_syntax.ML
changeset 69597 ff784d5a5bfb
parent 69593 3dda49e08b9d
child 74294 ee04dc00bf0a
--- a/src/ZF/ind_syntax.ML	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/ZF/ind_syntax.ML	Sat Jan 05 17:24:33 2019 +0100
@@ -23,10 +23,10 @@
 (*Creates All(%v.v:A --> P(v)) rather than Ball(A,P) *)
 fun mk_all_imp (A,P) =
     FOLogic.all_const iT $
-      Abs("v", iT, FOLogic.imp $ (@{const mem} $ Bound 0 $ A) $
+      Abs("v", iT, FOLogic.imp $ (\<^const>\<open>mem\<close> $ Bound 0 $ A) $
                    Term.betapply(P, Bound 0));
 
-fun mk_Collect (a, D, t) = @{const Collect} $ D $ absfree (a, iT) t;
+fun mk_Collect (a, D, t) = \<^const>\<open>Collect\<close> $ D $ absfree (a, iT) t;
 
 (*simple error-checking in the premises of an inductive definition*)
 fun chk_prem rec_hd (Const (\<^const_name>\<open>conj\<close>, _) $ _ $ _) =
@@ -83,20 +83,20 @@
       Logic.list_implies
         (map FOLogic.mk_Trueprop prems,
          FOLogic.mk_Trueprop
-            (@{const mem} $ list_comb (Const (Sign.full_bname sg name, T), args)
+            (\<^const>\<open>mem\<close> $ list_comb (Const (Sign.full_bname sg name, T), args)
                        $ rec_tm))
   in  map mk_intr constructs  end;
 
 fun mk_all_intr_tms sg arg = flat (ListPair.map (mk_intr_tms sg) arg);
 
-fun mk_Un (t1, t2) = @{const Un} $ t1 $ t2;
+fun mk_Un (t1, t2) = \<^const>\<open>Un\<close> $ t1 $ t2;
 
 (*Make a datatype's domain: form the union of its set parameters*)
 fun union_params (rec_tm, cs) =
   let val (_,args) = strip_comb rec_tm
       fun is_ind arg = (type_of arg = iT)
   in  case filter is_ind (args @ cs) of
-         [] => @{const zero}
+         [] => \<^const>\<open>zero\<close>
        | u_args => Balanced_Tree.make mk_Un u_args
   end;