removed needless comments
authorpaulson
Thu, 19 Aug 1999 15:13:37 +0200
changeset 7286 fcbf147e7b4c
parent 7285 52ea6848b908
child 7287 d603a06b30df
removed needless comments
TFL/tfl.sml
--- a/TFL/tfl.sml	Thu Aug 19 15:13:17 1999 +0200
+++ b/TFL/tfl.sml	Thu Aug 19 15:13:37 1999 +0200
@@ -493,10 +493,6 @@
      fun extract X = R.CONTEXT_REWRITE_RULE 
 	               (f, R1::SV, cut_apply, tflCongs@context_congs) X
  in {proto_def = proto_def,
-     (*LCP: want this??
-  (*Use == rather than = for definitions*)
-	 mk_const_def (Theory.sign_of thy) 
-	              (Name, Ty, S.rhs proto_def), *)
      SV=SV,
      WFR=WFR, 
      pats=pats,
@@ -516,7 +512,6 @@
 	   wfrec_eqns thy fid (congs tflCongs) eqns
      val R1 = S.rand WFR
      val f = #lhs(S.dest_eq proto_def)
-(*LCP: want this?     val f = #1 (Logic.dest_equals proto_def) *)
      val (extractants,TCl) = ListPair.unzip extracta
      val dummy = if !trace 
 		 then (writeln "Extractants = ";
@@ -537,13 +532,6 @@
      val (Name,Ty) = dest_atom c
      val defn = mk_const_def (Theory.sign_of thy) 
                  (Name, Ty, S.list_mk_abs (args,rhs)) 
-     (*LCP: want this??
-     val theory =
-       thy
-       |> PureThy.add_defs_i 
-            [Thm.no_attributes (fid ^ "_def", proto_def')];
-     val def = get_axiom theory (fid ^ "_def") RS meta_eq_to_obj_eq
-     *)
      val theory =
        thy
        |> PureThy.add_defs_i