src/HOL/ex/Predicate_Compile_ex.thy
changeset 32316 1d83ac469459
parent 32314 66bbad0bfef9
child 32317 b4b871808223
equal deleted inserted replaced
32315:79f324944be4 32316:1d83ac469459
    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}] *}
       
    75 setup {* fn thy => exception_trace (fn () => Predicate_Compile.add_quickcheck_equations [@{const_name tranclp}] thy)  *}
       
    76 
       
    77 thm tranclp.rpred_equation
       
    78 
    74 inductive succ :: "nat \<Rightarrow> nat \<Rightarrow> bool" where
    79 inductive succ :: "nat \<Rightarrow> nat \<Rightarrow> bool" where
    75     "succ 0 1"
    80     "succ 0 1"
    76   | "succ m n \<Longrightarrow> succ (Suc m) (Suc n)"
    81   | "succ m n \<Longrightarrow> succ (Suc m) (Suc n)"
    77 
    82 
    78 code_pred succ .
    83 code_pred succ .