equal
deleted
inserted
replaced
266 ] |
266 ] |
267 val to = NONE |
267 val to = NONE |
268 val th = Rewrite.rewrite_conv ctxt (pat, to) @{thms add.commute} ct |
268 val th = Rewrite.rewrite_conv ctxt (pat, to) @{thms add.commute} ct |
269 \<close> |
269 \<close> |
270 |
270 |
271 section \<open>Regression tests\<close> |
271 text \<open>Some regression tests\<close> |
272 |
272 |
273 ML \<open> |
273 ML \<open> |
274 val ct = \<^cterm>\<open>(\<lambda>b :: int. (\<lambda>a. b + a))\<close> |
274 val ct = \<^cterm>\<open>(\<lambda>b :: int. (\<lambda>a. b + a))\<close> |
275 val (x, ctxt) = yield_singleton Variable.add_fixes "x" \<^context> |
275 val (x, ctxt) = yield_singleton Variable.add_fixes "x" \<^context> |
276 val pat = [ |
276 val pat = [ |