src/HOL/HOLCF/Tools/Domain/domain_take_proofs.ML
changeset 69597 ff784d5a5bfb
parent 68236 b4484ec4a8f7
child 74305 28a582aa25dd
--- a/src/HOL/HOLCF/Tools/Domain/domain_take_proofs.ML	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/HOLCF/Tools/Domain/domain_take_proofs.ML	Sat Jan 05 17:24:33 2019 +0100
@@ -107,8 +107,8 @@
   }
 
 val beta_ss =
-  simpset_of (put_simpset HOL_basic_ss @{context}
-    addsimps @{thms simp_thms} addsimprocs [@{simproc beta_cfun_proc}])
+  simpset_of (put_simpset HOL_basic_ss \<^context>
+    addsimps @{thms simp_thms} addsimprocs [\<^simproc>\<open>beta_cfun_proc\<close>])
 
 (******************************************************************************)
 (******************************** theory data *********************************)
@@ -127,15 +127,15 @@
     Rec_Data.map (Symtab.insert (K true) (tname, bs))
 
 fun add_deflation_thm thm =
-    Context.theory_map (Named_Theorems.add_thm @{named_theorems domain_deflation} thm)
+    Context.theory_map (Named_Theorems.add_thm \<^named_theorems>\<open>domain_deflation\<close> thm)
 
 val get_rec_tab = Rec_Data.get
 fun get_deflation_thms thy =
-  rev (Named_Theorems.get (Proof_Context.init_global thy) @{named_theorems domain_deflation})
+  rev (Named_Theorems.get (Proof_Context.init_global thy) \<^named_theorems>\<open>domain_deflation\<close>)
 
-val map_ID_add = Named_Theorems.add @{named_theorems domain_map_ID}
+val map_ID_add = Named_Theorems.add \<^named_theorems>\<open>domain_map_ID\<close>
 fun get_map_ID_thms thy =
-  rev (Named_Theorems.get (Proof_Context.init_global thy) @{named_theorems domain_map_ID})
+  rev (Named_Theorems.get (Proof_Context.init_global thy) \<^named_theorems>\<open>domain_map_ID\<close>)
 
 
 (******************************************************************************)
@@ -149,7 +149,7 @@
 infix 9 `
 
 fun mk_deflation t =
-  Const (@{const_name deflation}, Term.fastype_of t --> boolT) $ t
+  Const (\<^const_name>\<open>deflation\<close>, Term.fastype_of t --> boolT) $ t
 
 fun mk_eqs (t, u) = HOLogic.mk_Trueprop (HOLogic.mk_eq (t, u))
 
@@ -272,7 +272,7 @@
     (* prove take_0 lemmas *)
     fun prove_take_0 ((take_const, dbind), (lhsT, _)) thy =
       let
-        val lhs = take_const $ @{term "0::nat"}
+        val lhs = take_const $ \<^term>\<open>0::nat\<close>
         val goal = mk_eqs (lhs, mk_bottom (lhsT ->> lhsT))
         val rules = take_defs @ @{thms iterate_0 fst_strict snd_strict}
         fun tac ctxt = simp_tac (put_simpset HOL_basic_ss ctxt addsimps rules) 1
@@ -289,7 +289,7 @@
     fun prove_take_Suc
           (((take_const, rep_abs), dbind), (_, rhsT)) thy =
       let
-        val lhs = take_const $ (@{term Suc} $ n)
+        val lhs = take_const $ (\<^term>\<open>Suc\<close> $ n)
         val body = map_of_typ thy (newTs ~~ take_is) rhsT
         val rhs = mk_cfcomp2 (rep_abs, body)
         val goal = mk_eqs (lhs, rhs)
@@ -434,9 +434,9 @@
         val iso_locale_thms = map iso_locale iso_infos
         val decisive_abs_rep_thms =
             map (fn x => @{thm decisive_abs_rep} OF [x]) iso_locale_thms
-        val n = Free ("n", @{typ nat})
+        val n = Free ("n", \<^typ>\<open>nat\<close>)
         fun mk_decisive t =
-            Const (@{const_name decisive}, fastype_of t --> boolT) $ t
+            Const (\<^const_name>\<open>decisive\<close>, fastype_of t --> boolT) $ t
         fun f take_const = mk_decisive (take_const $ n)
         val goal = mk_trp (foldr1 mk_conj (map f take_consts))
         val rules0 = @{thm decisive_bottom} :: take_0_thms
@@ -529,7 +529,7 @@
 
     (* test for finiteness of domain definitions *)
     local
-      val types = [@{type_name ssum}, @{type_name sprod}]
+      val types = [\<^type_name>\<open>ssum\<close>, \<^type_name>\<open>sprod\<close>]
       fun finite d T = if member (op =) absTs T then d else finite' d T
       and finite' d (Type (c, Ts)) =
           let val d' = d andalso member (op =) types c