src/Pure/drule.ML
changeset 59582 0fbed69ff081
parent 59058 a78612c67ec0
child 59586 ddf6deaadfe8
--- a/src/Pure/drule.ML	Tue Mar 03 19:08:04 2015 +0100
+++ b/src/Pure/drule.ML	Wed Mar 04 19:53:18 2015 +0100
@@ -130,7 +130,7 @@
   | _ => ct);
 
 (*The premises of a theorem, as a cterm list*)
-val cprems_of = strip_imp_prems o cprop_of;
+val cprems_of = strip_imp_prems o Thm.cprop_of;
 
 fun cterm_fun f ct = Thm.cterm_of (Thm.theory_of_cterm ct) (f (Thm.term_of ct));
 fun ctyp_fun f cT = Thm.ctyp_of (Thm.theory_of_ctyp cT) (f (Thm.typ_of cT));
@@ -168,7 +168,7 @@
 (*Beta-conversion for cterms, where x is an abstraction. Simply returns the rhs
   of the meta-equality returned by the beta_conversion rule.*)
 fun beta_conv x y =
-  Thm.dest_arg (cprop_of (Thm.beta_conversion false (Thm.apply x y)));
+  Thm.dest_arg (Thm.cprop_of (Thm.beta_conversion false (Thm.apply x y)));
 
 
 
@@ -406,8 +406,8 @@
 
 fun extensional eq =
   let val eq' =
-    Thm.abstract_rule "x" (Thm.dest_arg (fst (Thm.dest_equals (cprop_of eq)))) eq
-  in Thm.equal_elim (Thm.eta_conversion (cprop_of eq')) eq' end;
+    Thm.abstract_rule "x" (Thm.dest_arg (fst (Thm.dest_equals (Thm.cprop_of eq)))) eq
+  in Thm.equal_elim (Thm.eta_conversion (Thm.cprop_of eq')) eq' end;
 
 val equals_cong =
   store_standard_thm_open (Binding.make ("equals_cong", @{here}))
@@ -452,7 +452,7 @@
 fun binop_cong_rule ct th1 th2 = Thm.combination (arg_cong_rule ct th1) th2;
 
 local
-  val dest_eq = Thm.dest_equals o cprop_of
+  val dest_eq = Thm.dest_equals o Thm.cprop_of
   val rhs_of = snd o dest_eq
 in
 fun beta_eta_conversion t =
@@ -467,7 +467,7 @@
 
 (*Contract all eta-redexes in the theorem, lest they give rise to needless abstractions*)
 fun eta_contraction_rule th =
-  Thm.equal_elim (Thm.eta_conversion (cprop_of th)) th;
+  Thm.equal_elim (Thm.eta_conversion (Thm.cprop_of th)) th;
 
 
 (* abs_def *)
@@ -482,7 +482,7 @@
 
 fun contract_lhs th =
   Thm.transitive (Thm.symmetric (beta_eta_conversion
-    (fst (Thm.dest_equals (cprop_of th))))) th;
+    (fst (Thm.dest_equals (Thm.cprop_of th))))) th;
 
 fun var_args ct =
   (case try Thm.dest_comb ct of
@@ -793,7 +793,7 @@
   | cterm_instantiate ctpairs th =
       let
         val (thy, tye, _) = fold_rev add_types ctpairs (Thm.theory_of_thm th, Vartab.empty, 0);
-        val certT = ctyp_of thy;
+        val certT = Thm.ctyp_of thy;
         val instT =
           Vartab.fold (fn (xi, (S, T)) =>
             cons (certT (TVar (xi, S)), certT (Envir.norm_type tye T))) tye [];