src/HOL/ex/Predicate_Compile_ex.thy
changeset 32317 b4b871808223
parent 32316 1d83ac469459
child 32318 bca7fd849829
equal deleted inserted replaced
32316:1d83ac469459 32317:b4b871808223
    68   case tranclp
    68   case tranclp
    69   from this converse_tranclpE[OF this(1)] show thesis by metis
    69   from this converse_tranclpE[OF this(1)] show thesis by metis
    70 qed
    70 qed
    71 
    71 
    72 thm tranclp.equation
    72 thm tranclp.equation
    73 
    73 (*
    74 setup {* Predicate_Compile.add_sizelim_equations [@{const_name tranclp}] *}
    74 setup {* Predicate_Compile.add_sizelim_equations [@{const_name tranclp}] *}
    75 setup {* fn thy => exception_trace (fn () => Predicate_Compile.add_quickcheck_equations [@{const_name tranclp}] thy)  *}
    75 setup {* fn thy => exception_trace (fn () => Predicate_Compile.add_quickcheck_equations [@{const_name tranclp}] thy)  *}
    76 
    76 
    77 thm tranclp.rpred_equation
    77 thm tranclp.rpred_equation
    78 
    78 *)
    79 inductive succ :: "nat \<Rightarrow> nat \<Rightarrow> bool" where
    79 inductive succ :: "nat \<Rightarrow> nat \<Rightarrow> bool" where
    80     "succ 0 1"
    80     "succ 0 1"
    81   | "succ m n \<Longrightarrow> succ (Suc m) (Suc n)"
    81   | "succ m n \<Longrightarrow> succ (Suc m) (Suc n)"
    82 
    82 
    83 code_pred succ .
    83 code_pred succ .