src/HOL/Quickcheck_Examples/Quickcheck_Lattice_Examples.thy
changeset 80914 d97fdabd9e2b
parent 69597 ff784d5a5bfb
child 81132 dff7dfd8dce3
equal deleted inserted replaced
80913:46f59511b7bb 80914:d97fdabd9e2b
    11 
    11 
    12 text \<open>We show how other default types help to find counterexamples to propositions if
    12 text \<open>We show how other default types help to find counterexamples to propositions if
    13   the standard default type \<^typ>\<open>int\<close> is insufficient.\<close>
    13   the standard default type \<^typ>\<open>int\<close> is insufficient.\<close>
    14 
    14 
    15 notation
    15 notation
    16   less_eq  (infix "\<sqsubseteq>" 50) and
    16   less_eq  (infix \<open>\<sqsubseteq>\<close> 50) and
    17   less  (infix "\<sqsubset>" 50) and
    17   less  (infix \<open>\<sqsubset>\<close> 50) and
    18   top ("\<top>") and
    18   top (\<open>\<top>\<close>) and
    19   bot ("\<bottom>") and
    19   bot (\<open>\<bottom>\<close>) and
    20   inf (infixl "\<sqinter>" 70) and
    20   inf (infixl \<open>\<sqinter>\<close> 70) and
    21   sup (infixl "\<squnion>" 65)
    21   sup (infixl \<open>\<squnion>\<close> 65)
    22 
    22 
    23 declare [[quickcheck_narrowing_active = false, quickcheck_timeout = 3600]]
    23 declare [[quickcheck_narrowing_active = false, quickcheck_timeout = 3600]]
    24 
    24 
    25 subsection \<open>Distributive lattices\<close>
    25 subsection \<open>Distributive lattices\<close>
    26 
    26 
   131   quickcheck[expect = no_counterexample]
   131   quickcheck[expect = no_counterexample]
   132   by (simp add: eq_iff)
   132   by (simp add: eq_iff)
   133 
   133 
   134 
   134 
   135 no_notation
   135 no_notation
   136   less_eq  (infix "\<sqsubseteq>" 50) and
   136   less_eq  (infix \<open>\<sqsubseteq>\<close> 50) and
   137   less (infix "\<sqsubset>" 50) and
   137   less (infix \<open>\<sqsubset>\<close> 50) and
   138   inf  (infixl "\<sqinter>" 70) and
   138   inf  (infixl \<open>\<sqinter>\<close> 70) and
   139   sup  (infixl "\<squnion>" 65) and
   139   sup  (infixl \<open>\<squnion>\<close> 65) and
   140   top ("\<top>") and
   140   top (\<open>\<top>\<close>) and
   141   bot ("\<bottom>")
   141   bot (\<open>\<bottom>\<close>)
   142 
   142 
   143 end
   143 end