src/HOL/ex/Predicate_Compile_ex.thy
changeset 33146 bf852ef586f2
parent 33145 1a22f7ca1dfc
child 33147 180dc60bd88c
equal deleted inserted replaced
33145:1a22f7ca1dfc 33146:bf852ef586f2
    41 
    41 
    42 inductive append :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list \<Rightarrow> bool" where
    42 inductive append :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list \<Rightarrow> bool" where
    43     "append [] xs xs"
    43     "append [] xs xs"
    44   | "append xs ys zs \<Longrightarrow> append (x # xs) ys (x # zs)"
    44   | "append xs ys zs \<Longrightarrow> append (x # xs) ys (x # zs)"
    45 
    45 
    46 code_pred (mode: [1, 2], [3], [2, 3], [1, 3], [1, 2, 3]) [inductify] append .
    46 code_pred (mode: [1, 2], [3], [2, 3], [1, 3], [1, 2, 3]) append .
    47 code_pred [depth_limited] append .
    47 code_pred [depth_limited] append .
    48 code_pred [rpred] append .
    48 code_pred [rpred] append .
    49 
    49 
    50 thm append.equation
    50 thm append.equation
    51 thm append.depth_limited_equation
    51 thm append.depth_limited_equation
   364 
   364 
   365 code_pred [rpred] lexn .
   365 code_pred [rpred] lexn .
   366 
   366 
   367 thm lexn.rpred_equation
   367 thm lexn.rpred_equation
   368 
   368 
   369 code_pred [inductify] lenlex .
   369 code_pred [inductify, show_steps] lenlex .
   370 thm lenlex.equation
   370 thm lenlex.equation
   371 
   371 
   372 code_pred [inductify, rpred] lenlex .
   372 code_pred [inductify, rpred] lenlex .
   373 thm lenlex.rpred_equation
   373 thm lenlex.rpred_equation
   374 
   374 
   423 code_pred [inductify] rel_comp .
   423 code_pred [inductify] rel_comp .
   424 thm rel_comp.equation
   424 thm rel_comp.equation
   425 code_pred [inductify] Image .
   425 code_pred [inductify] Image .
   426 thm Image.equation
   426 thm Image.equation
   427 (*TODO: *)
   427 (*TODO: *)
   428 (*code_pred [inductify] Id_on .*)
   428 ML {* Toplevel.debug := true *}
       
   429 declare Id_on_def[unfolded UNION_def, code_pred_def]
       
   430 
       
   431 code_pred [inductify] Id_on .
       
   432 thm Id_on.equation
   429 code_pred [inductify] Domain .
   433 code_pred [inductify] Domain .
   430 thm Domain.equation
   434 thm Domain.equation
   431 code_pred [inductify] Range .
   435 code_pred [inductify] Range .
   432 thm sym_def
   436 thm sym_def
   433 code_pred [inductify] Field .
   437 code_pred [inductify] Field .
   434 (* code_pred [inductify] refl_on .*)
   438 declare Sigma_def[unfolded UNION_def, code_pred_def]
       
   439 declare refl_on_def[unfolded UNION_def, code_pred_def]
       
   440 code_pred [inductify] refl_on .
       
   441 thm refl_on.equation
   435 code_pred [inductify] total_on .
   442 code_pred [inductify] total_on .
   436 thm total_on.equation
   443 thm total_on.equation
   437 (*
   444 (*
   438 code_pred [inductify] sym .
   445 code_pred [inductify] sym .
   439 thm sym.equation
   446 thm sym.equation