changeset 366 | 06f044466f24 |
parent 361 | 8ba963a3e039 |
child 369 | 74ba778b09c9 |
365:718beb785213 | 366:06f044466f24 |
---|---|
1132 ML {* |
1132 ML {* |
1133 structure TacticData = ProofDataFun |
1133 structure TacticData = ProofDataFun |
1134 ( |
1134 ( |
1135 type T = thm list -> tactic; |
1135 type T = thm list -> tactic; |
1136 fun init _ = undefined; |
1136 fun init _ = undefined; |
1137 ); |
1137 ) |
1138 |
1138 |
1139 val set_tactic = TacticData.put; |
1139 val set_tactic = TacticData.put; |
1140 *} |
1140 *} |
1141 |
1141 |
1142 ML {* |
1142 ML {* |