src/HOL/Proofs/ex/XML_Data.thy
changeset 52630 fe411c1dc180
parent 52424 77075c576d4c
child 58372 bfd497f2f4c2
--- a/src/HOL/Proofs/ex/XML_Data.thy	Fri Jul 12 19:54:36 2013 +0200
+++ b/src/HOL/Proofs/ex/XML_Data.thy	Fri Jul 12 21:13:57 2013 +0200
@@ -1,47 +1,66 @@
 (*  Title:      HOL/Proofs/ex/XML_Data.thy
     Author:     Makarius
+    Author:     Stefan Berghofer
 
 XML data representation of proof terms.
 *)
 
 theory XML_Data
-imports Main
+imports "~~/src/HOL/Isar_Examples/Drinker"
 begin
 
 subsection {* Export and re-import of global proof terms *}
 
 ML {*
-  fun export_proof thm0 =
+  fun export_proof thm =
     let
-      val thy = Thm.theory_of_thm thm0;
-      val ctxt0 = Proof_Context.init_global thy;
-      val thy = Proof_Context.theory_of ctxt0;
-      val ((_, [thm]), ctxt) = Variable.import true [Thm.transfer thy thm0] ctxt0;
-
-      val prop = Thm.prop_of thm;  (* FIXME proper prop (wrt. import / strip) (!??) *)
+      val thy = Thm.theory_of_thm thm;
+      val {prop, hyps, shyps, ...} = Thm.rep_thm thm;
+      val (_, prop) = Logic.unconstrainT shyps (Logic.list_implies (hyps, prop));
       val prf =
-        Proofterm.proof_of (Proofterm.strip_thm (Thm.proof_body_of thm))
-        |> Proofterm.no_thm_proofs;
-    in XML.Encode.pair Term_XML.Encode.term Proofterm.encode (prop, prf) end;
+        Proofterm.proof_of (Proofterm.strip_thm (Thm.proof_body_of thm)) |>
+        Reconstruct.reconstruct_proof thy prop |>
+        Reconstruct.expand_proof thy [("", NONE)] |>
+        Proofterm.rew_proof thy |>
+        Proofterm.no_thm_proofs;
+    in Proofterm.encode prf end;
 
   fun import_proof thy xml =
     let
-      val (prop, prf) = XML.Decode.pair Term_XML.Decode.term Proofterm.decode xml;
-      val full_prf = Reconstruct.reconstruct_proof thy prop prf;
-    in Drule.export_without_context (Proof_Checker.thm_of_proof thy full_prf) end;
+      val prf = Proofterm.decode xml;
+      val (prf', _) = Proofterm.freeze_thaw_prf prf;
+    in Drule.export_without_context (Proof_Checker.thm_of_proof thy prf') end;
 *}
 
 
-subsection {* Example *}
+subsection {* Examples *}
 
 ML {* val thy1 = @{theory} *}
 
 lemma ex: "A \<longrightarrow> A" ..
 
-ML {*
+ML_val {*
   val xml = export_proof @{thm ex};
   val thm = import_proof thy1 xml;
 *}
 
+ML_val {*
+  val xml = export_proof @{thm de_Morgan};
+  val thm = import_proof thy1 xml;
+*}
+
+ML_val {*
+  val xml = export_proof @{thm Drinker's_Principle};
+  val thm = import_proof thy1 xml;
+*}
+
+text {* Some fairly large proof: *}
+
+ML_val {*
+  val xml = export_proof @{thm Int.times_int.abs_eq};
+  val thm = import_proof thy1 xml;
+  @{assert} (size (YXML.string_of_body xml) > 50000000);
+*}
+
 end