src/HOLCF/Tools/Domain/domain_theorems.ML
changeset 39557 fe5722fce758
parent 39288 f1ae2493d93f
child 40013 9db8fb58fddc
--- a/src/HOLCF/Tools/Domain/domain_theorems.ML	Mon Sep 20 15:29:53 2010 +0200
+++ b/src/HOLCF/Tools/Domain/domain_theorems.ML	Mon Sep 20 16:05:25 2010 +0200
@@ -124,7 +124,7 @@
 val rep_const = #rep_const iso_info;
 
 local
-  fun ga s dn = PureThy.get_thm thy (dn ^ "." ^ s);
+  fun ga s dn = Global_Theory.get_thm thy (dn ^ "." ^ s);
 in
   val ax_take_0      = ga "take_0" dname;
   val ax_take_strict = ga "take_strict" dname;
@@ -200,7 +200,7 @@
 
 in
   thy
-  |> PureThy.add_thmss [
+  |> Global_Theory.add_thmss [
      ((qualified "iso_rews"  , iso_rews    ), [simp]),
      ((qualified "nchotomy"  , [nchotomy]  ), []),
      ((qualified "exhaust"   , [exhaust]   ),
@@ -240,8 +240,8 @@
   val pg = pg' thy;
 
   local
-    fun ga s dn = PureThy.get_thm thy (dn ^ "." ^ s);
-    fun gts s dn = PureThy.get_thms thy (dn ^ "." ^ s);
+    fun ga s dn = Global_Theory.get_thm thy (dn ^ "." ^ s);
+    fun gts s dn = Global_Theory.get_thms thy (dn ^ "." ^ s);
   in
     val axs_rep_iso = map (ga "rep_iso") dnames;
     val axs_abs_iso = map (ga "abs_iso") dnames;
@@ -421,10 +421,10 @@
 
 in
   thy
-  |> snd o PureThy.add_thmss [
+  |> snd o Global_Theory.add_thmss [
      ((Binding.qualified true "finite_induct" comp_dbind, [finite_ind]), []),
      ((Binding.qualified true "induct"        comp_dbind, [ind]       ), [])]
-  |> (snd o PureThy.add_thmss (map ind_rule (dnames ~~ inducts)))
+  |> (snd o Global_Theory.add_thmss (map ind_rule (dnames ~~ inducts)))
 end; (* prove_induction *)
 
 (******************************************************************************)
@@ -444,7 +444,7 @@
 val n_eqs = length eqs;
 
 val take_rews =
-    maps (fn dn => PureThy.get_thms thy (dn ^ ".take_rews")) dnames;
+    maps (fn dn => Global_Theory.get_thms thy (dn ^ ".take_rews")) dnames;
 
 (* ----- define bisimulation predicate -------------------------------------- *)
 
@@ -465,7 +465,7 @@
       singleton (Syntax.check_terms (ProofContext.init_global thy)) (intern_term thy t);
   fun legacy_infer_prop thy t = legacy_infer_term thy (Type.constraint propT t);
   fun infer_props thy = map (apsnd (legacy_infer_prop thy));
-  fun add_defs_i x = PureThy.add_defs false (map Thm.no_attributes x);
+  fun add_defs_i x = Global_Theory.add_defs false (map Thm.no_attributes x);
   fun add_defs_infer defs thy = add_defs_i (infer_props thy defs) thy;
 
   fun one_con (con, args) =
@@ -568,7 +568,7 @@
     in pg [] goal (K tacs) end;
 end; (* local *)
 
-in thy |> snd o PureThy.add_thmss
+in thy |> snd o Global_Theory.add_thmss
     [((Binding.qualified true "coinduct" comp_dbind, [coind]), [])]
 end; (* let *)
 
@@ -603,7 +603,7 @@
 val take_lemmas = #take_lemma_thms take_info;
 
 val take_rews =
-    maps (fn dn => PureThy.get_thms thy (dn ^ ".take_rews")) dnames;
+    maps (fn dn => Global_Theory.get_thms thy (dn ^ ".take_rews")) dnames;
 
 (* prove induction rules, unless definition is indirect recursive *)
 val thy =