src/HOL/HOL.thy
changeset 33552 506f80a9afe8
parent 33523 96730ad673be
child 33756 47b7c9e0bf6e
equal deleted inserted replaced
33551:c40ced05b10a 33552:506f80a9afe8
  2001 
  2001 
  2002 subsubsection {* Quickcheck *}
  2002 subsubsection {* Quickcheck *}
  2003 
  2003 
  2004 quickcheck_params [size = 5, iterations = 50]
  2004 quickcheck_params [size = 5, iterations = 50]
  2005 
  2005 
  2006 ML {*
       
  2007 structure Quickcheck_RecFun_Simps = Named_Thms
       
  2008 (
       
  2009   val name = "quickcheck_recfun_simp"
       
  2010   val description = "simplification rules of recursive functions as needed by Quickcheck"
       
  2011 )
       
  2012 *}
       
  2013 
       
  2014 setup Quickcheck_RecFun_Simps.setup
       
  2015 
       
  2016 
  2006 
  2017 subsubsection {* Nitpick setup *}
  2007 subsubsection {* Nitpick setup *}
  2018 
  2008 
  2019 text {* This will be relocated once Nitpick is moved to HOL. *}
  2009 text {* This will be relocated once Nitpick is moved to HOL. *}
  2020 
  2010