Nominal/activities/tphols09/IDW/MW-Ex4.thy
author Christian Urban <urbanc@in.tum.de>
Thu, 13 Sep 2018 13:09:24 +0100 (2018-09-13)
changeset 539 5eaec0f9980f
parent 415 f1be8028a4a9
permissions -rw-r--r--
updated
theory Ex2
imports Main
begin

section {* Proof context data *}

ML {*
  structure My_Data = ProofDataFun(type T = int * string fun init _ = (2, "foo"))
*}

ML {* My_Data.get @{context} *}

ML {* val ctxt0 = @{context} *}
ML {* val ctxt1 = ctxt0 |> My_Data.map (fn (i, s) => (i + 1, s ^ "o")) *}
ML {* val ctxt2 = ctxt1 |> My_Data.map (fn (i, s) => (i + 1, s ^ "o")) *}

ML {* My_Data.get ctxt2 *}

end