src/HOL/ex/Quickcheck.thy
changeset 29579 cb520b766e00
parent 29132 3dac98ebae24
equal deleted inserted replaced
29578:8c4e961fcb08 29579:cb520b766e00
   198               val c = (fst o dest_Const o fst o strip_comb o fst
   198               val c = (fst o dest_Const o fst o strip_comb o fst
   199                 o HOLogic.dest_eq o HOLogic.dest_Trueprop o Thm.prop_of) thm;
   199                 o HOLogic.dest_eq o HOLogic.dest_Trueprop o Thm.prop_of) thm;
   200             in
   200             in
   201               lthy
   201               lthy
   202               |> LocalTheory.theory (Code.del_eqns c
   202               |> LocalTheory.theory (Code.del_eqns c
   203                    #> PureThy.add_thm ((fst (dest_Free random') ^ "_code", thm), [Thm.kind_internal])
   203                    #> PureThy.add_thm ((Binding.name (fst (dest_Free random') ^ "_code"), thm), [Thm.kind_internal])
   204                    #-> Code.add_eqn)
   204                    #-> Code.add_eqn)
   205             end;
   205             end;
   206         in
   206         in
   207           thy
   207           thy
   208           |> TheoryTarget.instantiation ([tyco], vs, @{sort random})
   208           |> TheoryTarget.instantiation ([tyco], vs, @{sort random})