Quot/Examples/IntEx.thy
changeset 908 1bf4337919d3
parent 875 cc951743c5e2
child 909 3e7a6ec549d1
equal deleted inserted replaced
907:e576a97e9a3e 908:1bf4337919d3
   184   and     c: "\<And>i. P i \<Longrightarrow> P (PLUS i (NEG ONE))"
   184   and     c: "\<And>i. P i \<Longrightarrow> P (PLUS i (NEG ONE))"
   185   shows      "P x"
   185   shows      "P x"
   186   using a b c
   186   using a b c
   187   by (lifting int_induct_raw)
   187   by (lifting int_induct_raw)
   188 
   188 
       
   189 lemma ex1tst: "\<exists>! (x :: nat \<times> nat) \<in> Respects (op \<approx>). True"
       
   190 sorry
       
   191 
       
   192 lemma ex1tst': "\<exists>! (x :: my_int). True"
       
   193 apply(lifting ex1tst)
       
   194 apply(cleaning)
       
   195 apply simp
       
   196 sorry
       
   197 
   189 lemma ho_tst: "foldl my_plus x [] = x"
   198 lemma ho_tst: "foldl my_plus x [] = x"
   190 apply simp
   199 apply simp
   191 done
   200 done
   192 
   201 
   193 
   202