equal
deleted
inserted
replaced
186 provides a richer reasoning infrastructure. The code of this package can be found in |
186 provides a richer reasoning infrastructure. The code of this package can be found in |
187 @{ML_file "HOL/Tools/inductive_package.ML"}. |
187 @{ML_file "HOL/Tools/inductive_package.ML"}. |
188 \end{readmore} |
188 \end{readmore} |
189 *} |
189 *} |
190 |
190 |
|
191 section {* Definitional Packages *} |
|
192 |
|
193 text {* Type declarations *} |
|
194 |
|
195 ML{*TypedefPackage.add_typedef false NONE (@{binding test},[],NoSyn) |
|
196 @{term "{1}::nat set"} NONE (simp_tac @{simpset} 1) @{theory} *} |
191 |
197 |
192 |
198 |
193 (*<*)end(*>*) |
199 (*<*)end(*>*) |