src/HOL/BNF_LFP.thy
changeset 56641 029997d3b5d8
parent 56640 0a35354137a5
child 56642 15cd15f9b40c
--- a/src/HOL/BNF_LFP.thy	Wed Apr 23 10:23:26 2014 +0200
+++ b/src/HOL/BNF_LFP.thy	Wed Apr 23 10:23:26 2014 +0200
@@ -218,6 +218,9 @@
 
 hide_fact (open) id_transfer
 
+datatype_new 'a i = I 'a
+thm i.size i.rec_o_map i.size_o_map
+
 datatype_new ('a, 'b) j = J0 | J 'a "('a, 'b) j"
 thm j.size j.rec_o_map j.size_o_map
 
@@ -249,11 +252,9 @@
 thm w.size w.rec_o_map w.size_o_map
 
 (*TODO:
-* deal with *unused* dead variables and other odd cases (e.g. recursion through fun)
 * what happens if recursion through arbitrary bnf, like 'fsize'?
   * by default
   * offer possibility to register size function and theorems
-* non-recursive types use 'case' instead of 'rec', causes trouble (revert?)
 * compat with old size?
   * recursion of old through new (e.g. through list)?
   * recursion of new through old?